Skip to content

Commit 7f2007a

Browse files
committed
chore(*): more since := in deprecated (#13723)
1 parent e956397 commit 7f2007a

File tree

23 files changed

+141
-140
lines changed

23 files changed

+141
-140
lines changed

Mathlib/Algebra/Algebra/Subalgebra/Basic.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -202,9 +202,8 @@ protected theorem intCast_mem {R : Type u} {A : Type v} [CommRing R] [Ring A] [A
202202
intCast_mem S n
203203
#align subalgebra.coe_int_mem Subalgebra.intCast_mem
204204

205-
-- 2024-04-05
206-
@[deprecated natCast_mem] alias coe_nat_mem := Subalgebra.natCast_mem
207-
@[deprecated intCast_mem] alias coe_int_mem := Subalgebra.intCast_mem
205+
@[deprecated natCast_mem (since := "2024-04-05")] alias coe_nat_mem := Subalgebra.natCast_mem
206+
@[deprecated intCast_mem (since := "2024-04-05")] alias coe_int_mem := Subalgebra.intCast_mem
208207

209208
/-- The projection from a subalgebra of `A` to an additive submonoid of `A`. -/
210209
def toAddSubmonoid {R : Type u} {A : Type v} [CommSemiring R] [Semiring A] [Algebra R A]

Mathlib/Algebra/BigOperators/Group/List.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -859,7 +859,7 @@ lemma unop_map_list_prod {F : Type*} [FunLike F M Nᵐᵒᵖ] [MonoidHomClass F
859859
namespace MonoidHom
860860

861861
/-- A morphism into the opposite monoid acts on the product by acting on the reversed elements. -/
862-
@[deprecated _root_.unop_map_list_prod]
862+
@[deprecated _root_.unop_map_list_prod (since := "2023-01-10")]
863863
protected theorem unop_map_list_prod (f : M →* Nᵐᵒᵖ) (l : List M) :
864864
(f l.prod).unop = (l.map (MulOpposite.unop ∘ f)).reverse.prod :=
865865
unop_map_list_prod f l

Mathlib/Algebra/GroupWithZero/Units/Basic.lean

Lines changed: 1 addition & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -579,9 +579,4 @@ noncomputable def commGroupWithZeroOfIsUnitOrEqZero [hM : CommMonoidWithZero M]
579579

580580
end NoncomputableDefs
581581

582-
-- 2024-03-20
583-
-- The names `div_mul_cancel`, `mul_div_cancel` and `mul_div_cancel_left` have been reused
584-
-- @[deprecated] alias div_mul_cancel := div_mul_cancel₀
585-
-- @[deprecated] alias mul_div_cancel := mul_div_cancel_right₀
586-
-- @[deprecated] alias mul_div_cancel_left := mul_div_cancel_left₀
587-
@[deprecated] alias mul_div_cancel' := mul_div_cancel₀
582+
@[deprecated (since := "2024-03-20")] alias mul_div_cancel' := mul_div_cancel₀

Mathlib/Algebra/Module/Defs.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -105,7 +105,7 @@ theorem two_smul : (2 : R) • x = x + x := by rw [← one_add_one_eq_two, add_s
105105
#align two_smul two_smul
106106

107107
set_option linter.deprecated false in
108-
@[deprecated]
108+
@[deprecated (since := "2022-12-31")]
109109
theorem two_smul' : (2 : R) • x = bit0 x :=
110110
two_smul R x
111111
#align two_smul' two_smul'

Mathlib/Algebra/Order/Field/Basic.lean

Lines changed: 4 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -293,11 +293,10 @@ lemma div_lt_div_of_pos_left (ha : 0 < a) (hc : 0 < c) (h : c < b) : a / b < a /
293293
simpa only [div_eq_mul_inv, mul_lt_mul_left ha, inv_lt_inv (hc.trans h) hc]
294294
#align div_lt_div_of_lt_left div_lt_div_of_pos_left
295295

296-
-- 2024-02-16
297-
@[deprecated] alias div_le_div_of_le_of_nonneg := div_le_div_of_nonneg_right
298-
@[deprecated] alias div_lt_div_of_lt := div_lt_div_of_pos_right
299-
@[deprecated] alias div_le_div_of_le_left := div_le_div_of_nonneg_left
300-
@[deprecated] alias div_lt_div_of_lt_left := div_lt_div_of_pos_left
296+
@[deprecated (since := "2024-02-16")] alias div_le_div_of_le_of_nonneg := div_le_div_of_nonneg_right
297+
@[deprecated (since := "2024-02-16")] alias div_lt_div_of_lt := div_lt_div_of_pos_right
298+
@[deprecated (since := "2024-02-16")] alias div_le_div_of_le_left := div_le_div_of_nonneg_left
299+
@[deprecated (since := "2024-02-16")] alias div_lt_div_of_lt_left := div_lt_div_of_pos_left
301300

302301
@[deprecated div_le_div_of_nonneg_right (since := "2024-02-16")]
303302
lemma div_le_div_of_le (hc : 0 ≤ c) (hab : a ≤ b) : a / c ≤ b / c :=

Mathlib/Algebra/Order/Floor.lean

Lines changed: 8 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -1741,11 +1741,14 @@ theorem natCast_ceil_eq_intCast_ceil (ha : 0 ≤ a) : (⌈a⌉₊ : α) = ⌈a
17411741
rw [← Int.ofNat_ceil_eq_ceil ha, Int.cast_natCast]
17421742
#align nat.cast_ceil_eq_cast_int_ceil natCast_ceil_eq_intCast_ceil
17431743

1744-
-- 2024-02-14
1745-
@[deprecated] alias Nat.cast_floor_eq_int_floor := Int.ofNat_floor_eq_floor
1746-
@[deprecated] alias Nat.cast_ceil_eq_int_ceil := Int.ofNat_ceil_eq_ceil
1747-
@[deprecated] alias Nat.cast_floor_eq_cast_int_floor := natCast_floor_eq_intCast_floor
1748-
@[deprecated] alias Nat.cast_ceil_eq_cast_int_ceil := natCast_ceil_eq_intCast_ceil
1744+
@[deprecated (since := "2024-02-14")] alias Nat.cast_floor_eq_int_floor := Int.ofNat_floor_eq_floor
1745+
@[deprecated (since := "2024-02-14")] alias Nat.cast_ceil_eq_int_ceil := Int.ofNat_ceil_eq_ceil
1746+
1747+
@[deprecated (since := "2024-02-14")]
1748+
alias Nat.cast_floor_eq_cast_int_floor := natCast_floor_eq_intCast_floor
1749+
1750+
@[deprecated (since := "2024-02-14")]
1751+
alias Nat.cast_ceil_eq_cast_int_ceil := natCast_ceil_eq_intCast_ceil
17491752

17501753
end FloorRingToSemiring
17511754

Mathlib/Algebra/Order/Monoid/Defs.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -118,8 +118,8 @@ instance (priority := 100) OrderedCancelCommMonoid.toCancelCommMonoid : CancelCo
118118
end OrderedCancelCommMonoid
119119

120120
set_option linter.deprecated false in
121-
@[deprecated] theorem bit0_pos [OrderedAddCommMonoid α] {a : α} (h : 0 < a) : 0 < bit0 a :=
122-
add_pos' h h
121+
@[deprecated (since := "2022-11-28")]
122+
theorem bit0_pos [OrderedAddCommMonoid α] {a : α} (h : 0 < a) : 0 < bit0 a := add_pos' h h
123123
#align bit0_pos bit0_pos
124124

125125
/-- A linearly ordered additive commutative monoid. -/

Mathlib/Algebra/Order/Monoid/Unbundled/Basic.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -1695,12 +1695,12 @@ section Bit
16951695
set_option linter.deprecated false
16961696
variable [Add α] [Preorder α]
16971697

1698-
@[deprecated]
1698+
@[deprecated (since := "2022-11-20")]
16991699
theorem bit0_mono [CovariantClass α α (· + ·) (· ≤ ·)] [CovariantClass α α (swap (· + ·)) (· ≤ ·)] :
17001700
Monotone (bit0 : α → α) := fun _ _ h => add_le_add h h
17011701
#align bit0_mono bit0_mono
17021702

1703-
@[deprecated]
1703+
@[deprecated (since := "2022-11-20")]
17041704
theorem bit0_strictMono [CovariantClass α α (· + ·) (· < ·)]
17051705
[CovariantClass α α (swap (· + ·)) (· < ·)] :
17061706
StrictMono (bit0 : α → α) := fun _ _ h => add_lt_add h h

Mathlib/Algebra/Order/Monoid/WithTop.lean

Lines changed: 6 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -369,10 +369,9 @@ instance addMonoidWithOne : AddMonoidWithOne (WithTop α) :=
369369
@[simp] lemma top_ne_natCast (n : ℕ) : (⊤ : WithTop α) ≠ n := top_ne_coe
370370
#align with_top.top_ne_nat WithTop.top_ne_natCast
371371

372-
-- 2024-04-05
373-
@[deprecated] alias coe_nat := coe_natCast
374-
@[deprecated] alias nat_ne_top := natCast_ne_top
375-
@[deprecated] alias top_ne_nat := top_ne_natCast
372+
@[deprecated (since := "2024-04-05")] alias coe_nat := coe_natCast
373+
@[deprecated (since := "2024-04-05")] alias nat_ne_top := natCast_ne_top
374+
@[deprecated (since := "2024-04-05")] alias top_ne_nat := top_ne_natCast
376375

377376
end AddMonoidWithOne
378377

@@ -570,10 +569,9 @@ instance addMonoidWithOne : AddMonoidWithOne (WithBot α) := WithTop.addMonoidWi
570569
@[simp] lemma bot_ne_natCast (n : ℕ) : (⊥ : WithBot α) ≠ n := bot_ne_coe
571570
#align with_bot.bot_ne_nat WithBot.bot_ne_natCast
572571

573-
-- 2024-04-05
574-
@[deprecated] alias coe_nat := coe_natCast
575-
@[deprecated] alias nat_ne_bot := natCast_ne_bot
576-
@[deprecated] alias bot_ne_nat := bot_ne_natCast
572+
@[deprecated (since := "2024-04-05")] alias coe_nat := coe_natCast
573+
@[deprecated (since := "2024-04-05")] alias nat_ne_bot := natCast_ne_bot
574+
@[deprecated (since := "2024-04-05")] alias bot_ne_nat := bot_ne_natCast
577575

578576
end AddMonoidWithOne
579577

Mathlib/Algebra/Order/Ring/Basic.lean

Lines changed: 26 additions & 20 deletions
Original file line numberDiff line numberDiff line change
@@ -438,23 +438,29 @@ end LinearOrderedSemiring
438438
Those lemmas have been deprecated on 2023-12-23.
439439
-/
440440

441-
@[deprecated] alias pow_mono := pow_right_mono
442-
@[deprecated] alias pow_le_pow := pow_le_pow_right
443-
@[deprecated] alias pow_le_pow_of_le_left := pow_le_pow_left
444-
@[deprecated] alias pow_lt_pow_of_lt_left := pow_lt_pow_left
445-
@[deprecated] alias strictMonoOn_pow := pow_left_strictMonoOn
446-
@[deprecated] alias pow_strictMono_right := pow_right_strictMono
447-
@[deprecated] alias pow_lt_pow := pow_lt_pow_right
448-
@[deprecated] alias pow_lt_pow_iff := pow_lt_pow_iff_right
449-
@[deprecated] alias pow_le_pow_iff := pow_le_pow_iff_right
450-
@[deprecated] alias self_lt_pow := lt_self_pow
451-
@[deprecated] alias strictAnti_pow := pow_right_strictAnti
452-
@[deprecated] alias pow_lt_pow_iff_of_lt_one := pow_lt_pow_iff_right_of_lt_one
453-
@[deprecated] alias pow_lt_pow_of_lt_one := pow_lt_pow_right_of_lt_one
454-
@[deprecated] alias lt_of_pow_lt_pow := lt_of_pow_lt_pow_left
455-
@[deprecated] alias le_of_pow_le_pow := le_of_pow_le_pow_left
456-
@[deprecated] alias self_le_pow := le_self_pow
457-
@[deprecated] alias Nat.pow_lt_pow_of_lt_right := pow_lt_pow_right
458-
@[deprecated] protected alias Nat.pow_right_strictMono := pow_right_strictMono
459-
@[deprecated] alias Nat.pow_le_iff_le_right := pow_le_pow_iff_right
460-
@[deprecated] alias Nat.pow_lt_iff_lt_right := pow_lt_pow_iff_right
441+
@[deprecated (since := "2023-12-23")] alias pow_mono := pow_right_mono
442+
@[deprecated (since := "2023-12-23")] alias pow_le_pow := pow_le_pow_right
443+
@[deprecated (since := "2023-12-23")] alias pow_le_pow_of_le_left := pow_le_pow_left
444+
@[deprecated (since := "2023-12-23")] alias pow_lt_pow_of_lt_left := pow_lt_pow_left
445+
@[deprecated (since := "2023-12-23")] alias strictMonoOn_pow := pow_left_strictMonoOn
446+
@[deprecated (since := "2023-12-23")] alias pow_strictMono_right := pow_right_strictMono
447+
@[deprecated (since := "2023-12-23")] alias pow_lt_pow := pow_lt_pow_right
448+
@[deprecated (since := "2023-12-23")] alias pow_lt_pow_iff := pow_lt_pow_iff_right
449+
@[deprecated (since := "2023-12-23")] alias pow_le_pow_iff := pow_le_pow_iff_right
450+
@[deprecated (since := "2023-12-23")] alias self_lt_pow := lt_self_pow
451+
@[deprecated (since := "2023-12-23")] alias strictAnti_pow := pow_right_strictAnti
452+
453+
@[deprecated (since := "2023-12-23")]
454+
alias pow_lt_pow_iff_of_lt_one := pow_lt_pow_iff_right_of_lt_one
455+
456+
@[deprecated (since := "2023-12-23")] alias pow_lt_pow_of_lt_one := pow_lt_pow_right_of_lt_one
457+
@[deprecated (since := "2023-12-23")] alias lt_of_pow_lt_pow := lt_of_pow_lt_pow_left
458+
@[deprecated (since := "2023-12-23")] alias le_of_pow_le_pow := le_of_pow_le_pow_left
459+
@[deprecated (since := "2023-12-23")] alias self_le_pow := le_self_pow
460+
@[deprecated (since := "2023-12-23")] alias Nat.pow_lt_pow_of_lt_right := pow_lt_pow_right
461+
462+
@[deprecated (since := "2023-12-23")]
463+
protected alias Nat.pow_right_strictMono := pow_right_strictMono
464+
465+
@[deprecated (since := "2023-12-23")] alias Nat.pow_le_iff_le_right := pow_le_pow_iff_right
466+
@[deprecated (since := "2023-12-23")] alias Nat.pow_lt_iff_lt_right := pow_lt_pow_iff_right

0 commit comments

Comments
 (0)