Skip to content

Commit 3877b4e

Browse files
committed
document move
1 parent de6aeda commit 3877b4e

File tree

1 file changed

+2
-0
lines changed

1 file changed

+2
-0
lines changed

src/Std/Classes/Ord/Basic.lean

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -332,11 +332,13 @@ theorem LawfulEqCmp.compare_eq_iff_eq {a b : α} : cmp a b = .eq ↔ a = b :=
332332
theorem 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]
336337
theorem 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]
341343
theorem LawfulEqOrd.compare_beq_iff_eq [Ord α] [LawfulEqOrd α] {a b : α} :
342344
compare a b == .eq ↔ a = b :=

0 commit comments

Comments
 (0)