We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
gt_irrefl
1 parent cb99f5a commit b2b0027Copy full SHA for b2b0027
Mathlib/Order/Defs/PartialOrder.lean
@@ -81,7 +81,8 @@ alias LE.le.not_gt := not_lt_of_ge
81
lemma ge_trans : a ≥ b → b ≥ c → a ≥ c := fun h₁ h₂ => le_trans h₂ h₁
82
83
lemma lt_irrefl (a : α) : ¬a < a := fun h ↦ not_le_of_gt h le_rfl
84
-lemma gt_irrefl (a : α) : ¬a > a := lt_irrefl _
+
85
+@[deprecated (since := "2025-06-07")] alias gt_irrefl := lt_irrefl
86
87
lemma lt_of_lt_of_le (hab : a < b) (hbc : b ≤ c) : a < c :=
88
lt_of_le_not_ge (le_trans (le_of_lt hab) hbc) fun hca ↦ not_le_of_gt hab (le_trans hbc hca)
0 commit comments