File tree Expand file tree Collapse file tree 1 file changed +2
-0
lines changed
Expand file tree Collapse file tree 1 file changed +2
-0
lines changed Original file line number Diff line number Diff line change @@ -332,11 +332,13 @@ theorem LawfulEqCmp.compare_eq_iff_eq {a b : α} : cmp a b = .eq ↔ a = b :=
332332theorem LawfulEqCmp.compare_beq_iff_eq {a b : α} : cmp a b == .eq ↔ a = b :=
333333 beq_iff_eq.trans compare_eq_iff_eq
334334
335+ /-- The corresponding lemma for `LawfulEqCmp` is `LawfulEqCmp.compare_eq_iff_eq` -/
335336@[simp, grind]
336337theorem LawfulEqOrd.compare_eq_iff_eq [Ord α] [LawfulEqOrd α] {a b : α} :
337338 compare a b = .eq ↔ a = b :=
338339 LawfulEqCmp.compare_eq_iff_eq
339340
341+ /-- The corresponding lemma for `LawfulEqCmp` is `LawfulEqCmp.compare_beq_iff_eq` -/
340342@[simp, grind]
341343theorem LawfulEqOrd.compare_beq_iff_eq [Ord α] [LawfulEqOrd α] {a b : α} :
342344 compare a b == .eq ↔ a = b :=
You can’t perform that action at this time.
0 commit comments