Skip to content

Commit b2b0027

Browse files
committed
chore(Order): deprecate gt_irrefl (#25567)
1 parent cb99f5a commit b2b0027

File tree

1 file changed

+2
-1
lines changed

1 file changed

+2
-1
lines changed

Mathlib/Order/Defs/PartialOrder.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -81,7 +81,8 @@ alias LE.le.not_gt := not_lt_of_ge
8181
lemma ge_trans : a ≥ b → b ≥ c → a ≥ c := fun h₁ h₂ => le_trans h₂ h₁
8282

8383
lemma lt_irrefl (a : α) : ¬a < a := fun h ↦ not_le_of_gt h le_rfl
84-
lemma gt_irrefl (a : α) : ¬a > a := lt_irrefl _
84+
85+
@[deprecated (since := "2025-06-07")] alias gt_irrefl := lt_irrefl
8586

8687
lemma lt_of_lt_of_le (hab : a < b) (hbc : b ≤ c) : a < c :=
8788
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

Comments
 (0)