Skip to content

Commit e3ed192

Browse files
committed
chore: remove >6 months old deprecations (#22996)
1 parent 1f09ac5 commit e3ed192

File tree

5 files changed

+0
-63
lines changed

5 files changed

+0
-63
lines changed

Mathlib/Order/WithBot.lean

Lines changed: 0 additions & 39 deletions
Original file line numberDiff line numberDiff line change
@@ -207,15 +207,6 @@ lemma not_coe_le_bot (a : α) : ¬(a : WithBot α) ≤ ⊥ := by simp [le_def]
207207

208208
instance orderBot : OrderBot (WithBot α) where bot_le := by simp [le_def]
209209

210-
-- TODO: This deprecated lemma is still used (through simp)
211-
@[simp, deprecated coe_le_coe "Don't mix Option and WithBot" (since := "2024-05-27")]
212-
theorem some_le_some : @LE.le (WithBot α) _ (Option.some a) (Option.some b) ↔ a ≤ b :=
213-
coe_le_coe
214-
215-
-- TODO: This deprecated lemma is still used (through simp)
216-
@[simp, deprecated bot_le "Don't mix Option and WithBot" (since := "2024-05-27")]
217-
theorem none_le {a : WithBot α} : @LE.le (WithBot α) _ none a := bot_le
218-
219210
instance orderTop [OrderTop α] : OrderTop (WithBot α) where le_top x := by cases x <;> simp [le_def]
220211

221212
instance instBoundedOrder [OrderTop α] : BoundedOrder (WithBot α) :=
@@ -258,18 +249,6 @@ lemma lt_def : x < y ↔ ∃ b : α, y = ↑b ∧ ∀ a : α, x = ↑a → a < b
258249
@[simp] lemma bot_lt_coe (a : α) : ⊥ < (a : WithBot α) := by simp [lt_def]
259250
@[simp] protected lemma not_lt_bot (a : WithBot α) : ¬a < ⊥ := by simp [lt_def]
260251

261-
-- TODO: This deprecated lemma is still used (through simp)
262-
@[simp, deprecated coe_lt_coe "Don't mix Option and WithBot" (since := "2024-05-27")]
263-
theorem some_lt_some : @LT.lt (WithBot α) _ (Option.some a) (Option.some b) ↔ a < b := coe_lt_coe
264-
265-
-- TODO: This deprecated lemma is still used (through simp)
266-
@[simp, deprecated bot_lt_coe "Don't mix Option and WithBot" (since := "2024-05-27")]
267-
theorem none_lt_some (a : α) : @LT.lt (WithBot α) _ none (some a) := bot_lt_coe _
268-
269-
-- TODO: This deprecated lemma is still used (through simp)
270-
@[simp, deprecated not_lt_bot "Don't mix Option and WithBot" (since := "2024-05-27")]
271-
theorem not_lt_none (a : WithBot α) : ¬@LT.lt (WithBot α) _ a none := WithBot.not_lt_bot _
272-
273252
lemma lt_iff_exists_coe : x < y ↔ ∃ b : α, y = b ∧ x < b := by cases y <;> simp
274253

275254
lemma lt_coe_iff : x < b ↔ ∀ a : α, x = a → a < b := by simp [lt_def]
@@ -709,17 +688,8 @@ lemma le_def : x ≤ y ↔ ∀ b : α, y = ↑b → ∃ a : α, x = ↑a ∧ a
709688

710689
lemma not_top_le_coe (a : α) : ¬ ⊤ ≤ (a : WithTop α) := by simp [le_def]
711690

712-
-- TODO: This deprecated lemma is still used (through simp)
713-
@[simp, deprecated coe_le_coe "Don't mix Option and WithTop" (since := "2024-05-27")]
714-
theorem some_le_some : @LE.le (WithTop α) _ (Option.some a) (Option.some b) ↔ a ≤ b :=
715-
coe_le_coe
716-
717691
instance orderTop : OrderTop (WithTop α) where le_top := by simp [le_def]
718692

719-
-- TODO: This deprecated lemma is still used (through simp)
720-
@[simp, deprecated le_top "Don't mix Option and WithTop" (since := "2024-05-27")]
721-
theorem le_none {a : WithTop α} : @LE.le (WithTop α) _ a none := le_top
722-
723693
instance orderBot [OrderBot α] : OrderBot (WithTop α) where bot_le x := by cases x <;> simp [le_def]
724694

725695
instance boundedOrder [OrderBot α] : BoundedOrder (WithTop α) :=
@@ -762,15 +732,6 @@ lemma lt_def : x < y ↔ ∃ a : α, x = ↑a ∧ ∀ b : α, y = ↑b → a < b
762732
@[simp] lemma coe_lt_top (a : α) : (a : WithTop α) < ⊤ := by simp [lt_def]
763733
@[simp] protected lemma not_top_lt (a : WithTop α) : ¬⊤ < a := by simp [lt_def]
764734

765-
@[simp, deprecated coe_lt_coe "Don't mix Option and WithTop" (since := "2024-05-27")]
766-
theorem some_lt_some : @LT.lt (WithTop α) _ (Option.some a) (Option.some b) ↔ a < b := coe_lt_coe
767-
768-
@[simp, deprecated coe_lt_top "Don't mix Option and WithTop" (since := "2024-05-27")]
769-
theorem some_lt_none (a : α) : @LT.lt (WithTop α) _ (Option.some a) none := coe_lt_top a
770-
771-
@[simp, deprecated not_top_lt "Don't mix Option and WithTop" (since := "2024-05-27")]
772-
theorem not_none_lt (a : WithTop α) : ¬@LT.lt (WithTop α) _ none a := WithTop.not_top_lt _
773-
774735
lemma lt_iff_exists_coe : x < y ↔ ∃ a : α, x = a ∧ a < y := by cases x <;> simp
775736

776737
lemma coe_lt_iff : a < y ↔ ∀ b : α, y = b → a < b := by simp [lt_def]

Mathlib/SetTheory/Cardinal/Regular.lean

Lines changed: 0 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -121,22 +121,10 @@ theorem iSup_lt_ord_lift_of_isRegular {ι} {f : ι → Ordinal} {c} (hc : IsRegu
121121
(hι : Cardinal.lift.{v, u} #ι < c) : (∀ i, f i < c.ord) → iSup f < c.ord :=
122122
iSup_lt_ord_lift (by rwa [hc.cof_eq])
123123

124-
set_option linter.deprecated false in
125-
@[deprecated iSup_lt_ord_lift_of_isRegular (since := "2024-08-27")]
126-
theorem sup_lt_ord_lift_of_isRegular {ι} {f : ι → Ordinal} {c} (hc : IsRegular c)
127-
(hι : Cardinal.lift.{v, u} #ι < c) : (∀ i, f i < c.ord) → Ordinal.sup.{u, v} f < c.ord :=
128-
iSup_lt_ord_lift_of_isRegular hc hι
129-
130124
theorem iSup_lt_ord_of_isRegular {ι} {f : ι → Ordinal} {c} (hc : IsRegular c) (hι : #ι < c) :
131125
(∀ i, f i < c.ord) → iSup f < c.ord :=
132126
iSup_lt_ord (by rwa [hc.cof_eq])
133127

134-
set_option linter.deprecated false in
135-
@[deprecated iSup_lt_ord_of_isRegular (since := "2024-08-27")]
136-
theorem sup_lt_ord_of_isRegular {ι} {f : ι → Ordinal} {c} (hc : IsRegular c) (hι : #ι < c) :
137-
(∀ i, f i < c.ord) → Ordinal.sup f < c.ord :=
138-
iSup_lt_ord_of_isRegular hc hι
139-
140128
theorem blsub_lt_ord_lift_of_isRegular {o : Ordinal} {f : ∀ a < o, Ordinal} {c} (hc : IsRegular c)
141129
(ho : Cardinal.lift.{v, u} o.card < c) :
142130
(∀ i hi, f i hi < c.ord) → Ordinal.blsub.{u, v} o f < c.ord :=

Mathlib/SetTheory/Ordinal/Arithmetic.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -344,9 +344,6 @@ theorem has_succ_of_type_succ_lt {α} {r : α → α → Prop} [wo : IsWellOrder
344344
theorem toType_noMax_of_succ_lt {o : Ordinal} (ho : ∀ a < o, succ a < o) : NoMaxOrder o.toType :=
345345
⟨has_succ_of_type_succ_lt (type_toType _ ▸ ho)⟩
346346

347-
@[deprecated toType_noMax_of_succ_lt (since := "2024-08-26")]
348-
alias out_no_max_of_succ_lt := toType_noMax_of_succ_lt
349-
350347
theorem bounded_singleton {r : α → α → Prop} [IsWellOrder α r] (hr : (type r).IsLimit) (x) :
351348
Bounded r {x} := by
352349
refine ⟨enum r ⟨succ (typein r x), hr.succ_lt (typein_lt_type r x)⟩, ?_⟩

Mathlib/SetTheory/Ordinal/FixedPoint.lean

Lines changed: 0 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -462,9 +462,6 @@ theorem lt_nfp_iff {a b} : a < nfp f b ↔ ∃ n, a < f^[n] b := by
462462
rw [← iSup_iterate_eq_nfp]
463463
exact Ordinal.lt_iSup_iff
464464

465-
@[deprecated lt_nfp_iff (since := "2024-02-16")]
466-
alias lt_nfp := lt_nfp_iff
467-
468465
theorem nfp_le_iff {a b} : nfp f a ≤ b ↔ ∀ n, f^[n] a ≤ b := by
469466
rw [← iSup_iterate_eq_nfp]
470467
exact Ordinal.iSup_le_iff

Mathlib/SetTheory/Ordinal/NaturalOps.lean

Lines changed: 0 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -377,9 +377,6 @@ instance : CharZero NatOrdinal where
377377
apply_fun toOrdinal at h
378378
simpa using h
379379

380-
@[deprecated toOrdinal_natCast (since := "2024-03-05")]
381-
alias toOrdinal_cast_nat := toOrdinal_natCast
382-
383380
end NatOrdinal
384381

385382
open NatOrdinal
@@ -396,9 +393,6 @@ theorem toNatOrdinal_natCast (n : ℕ) : toNatOrdinal n = n := by
396393
rw [← toOrdinal_natCast n]
397394
rfl
398395

399-
@[deprecated toNatOrdinal_natCast (since := "2024-03-05")]
400-
alias toNatOrdinal_cast_nat := toNatOrdinal_natCast
401-
402396
theorem lt_of_nadd_lt_nadd_left : ∀ {a b c}, a ♯ b < a ♯ c → b < c :=
403397
@lt_of_add_lt_add_left NatOrdinal _ _ _
404398

0 commit comments

Comments
 (0)