Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 40d2b50

Browse files
committed
fix(algebra/order): update to lean
The new `not_lt_of_lt` in core is not substitutable for this one because it is in the new algebraic hierarchy and mathlib is still on the old one. But this isn't used anywhere, so I'll just remove it instead of renaming.
1 parent f467c81 commit 40d2b50

File tree

1 file changed

+0
-3
lines changed

1 file changed

+0
-3
lines changed

algebra/order.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -12,9 +12,6 @@ lemma not_le_of_lt [preorder α] {a b : α} (h : a < b) : ¬ b ≤ a :=
1212

1313
lemma not_lt_of_le [preorder α] {a b : α} (h : a ≤ b) : ¬ b < a
1414
| hab := not_le_of_gt hab h
15-
16-
lemma not_lt_of_lt [linear_order α] {a b : α} (h : a < b) : ¬ b < a :=
17-
lt_asymm h
1815

1916
lemma le_iff_eq_or_lt [partial_order α] {a b : α} : a ≤ b ↔ a = b ∨ a < b :=
2017
le_iff_lt_or_eq.trans or.comm

0 commit comments

Comments
 (0)