File tree Expand file tree Collapse file tree 1 file changed +14
-0
lines changed Expand file tree Collapse file tree 1 file changed +14
-0
lines changed Original file line number Diff line number Diff line change @@ -117,6 +117,10 @@ theorem lt_of_eq_of_lt' : b = c → a < b → a < c :=
117
117
theorem not_lt_iff_not_le_or_ge : ¬a < b ↔ ¬a ≤ b ∨ b ≤ a := by
118
118
rw [lt_iff_le_not_le, Classical.not_and_iff_not_or_not, Classical.not_not]
119
119
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
+
120
124
/-- If `x = y` then `y ≤ x`. Note: this lemma uses `y ≤ x` instead of `x ≥ y`, because `le` is used
121
125
almost exclusively in mathlib. -/
122
126
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
206
210
alias LE.le.lt_of_ne' := lt_of_le_of_ne'
207
211
alias LE.le.lt_or_eq := lt_or_eq_of_le
208
212
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
+
209
223
namespace LE.le
210
224
211
225
theorem lt_iff_ne (h : a ≤ b) : a < b ↔ a ≠ b :=
You can’t perform that action at this time.
0 commit comments