Skip to content

Commit 3a141dd

Browse files
committed
feat: ¬ a < b ↔ a ≤ b → b ≤ a (#23737)
... and other lemmas that are useful to link the various definitions of minimality of an element.
1 parent da7280f commit 3a141dd

File tree

1 file changed

+14
-0
lines changed

1 file changed

+14
-0
lines changed

Mathlib/Order/Basic.lean

Lines changed: 14 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -117,6 +117,10 @@ theorem lt_of_eq_of_lt' : b = c → a < b → a < c :=
117117
theorem not_lt_iff_not_le_or_ge : ¬a < b ↔ ¬a ≤ b ∨ b ≤ a := by
118118
rw [lt_iff_le_not_le, Classical.not_and_iff_not_or_not, Classical.not_not]
119119

120+
-- Unnecessary brackets are here for readability
121+
lemma not_lt_iff_le_imp_le : ¬ a < b ↔ (a ≤ b → b ≤ a) := by
122+
simp [not_lt_iff_not_le_or_ge, or_iff_not_imp_left]
123+
120124
/-- If `x = y` then `y ≤ x`. Note: this lemma uses `y ≤ x` instead of `x ≥ y`, because `le` is used
121125
almost exclusively in mathlib. -/
122126
lemma ge_of_eq (h : a = b) : b ≤ a := le_of_eq h.symm
@@ -206,6 +210,16 @@ alias LE.le.lt_of_ne := lt_of_le_of_ne
206210
alias LE.le.lt_of_ne' := lt_of_le_of_ne'
207211
alias LE.le.lt_or_eq := lt_or_eq_of_le
208212

213+
-- Unnecessary brackets are here for readability
214+
lemma le_imp_eq_iff_le_imp_le : (a ≤ b → b = a) ↔ (a ≤ b → b ≤ a) where
215+
mp h hab := (h hab).le
216+
mpr h hab := (h hab).antisymm hab
217+
218+
-- Unnecessary brackets are here for readability
219+
lemma ge_imp_eq_iff_le_imp_le : (a ≤ b → a = b) ↔ (a ≤ b → b ≤ a) where
220+
mp h hab := (h hab).ge
221+
mpr h hab := hab.antisymm (h hab)
222+
209223
namespace LE.le
210224

211225
theorem lt_iff_ne (h : a ≤ b) : a < b ↔ a ≠ b :=

0 commit comments

Comments
 (0)