Skip to content

Commit 38c3948

Browse files
authored
chore: add missing deprecation dates (#5884)
1 parent 09802e8 commit 38c3948

File tree

6 files changed

+18
-18
lines changed

6 files changed

+18
-18
lines changed

src/Init/Data/BitVec/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -1792,7 +1792,7 @@ theorem setWidth_succ (x : BitVec w) :
17921792
· simp_all
17931793
· omega
17941794

1795-
@[deprecated "Use the reverse direction of `cons_msb_setWidth`"]
1795+
@[deprecated "Use the reverse direction of `cons_msb_setWidth`" (since := "2024-09-23")]
17961796
theorem eq_msb_cons_setWidth (x : BitVec (w+1)) : x = (cons x.msb (x.setWidth w)) := by
17971797
simp
17981798

src/Init/PropLemmas.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -643,11 +643,11 @@ theorem decide_ite (u : Prop) [du : Decidable u] (p q : Prop)
643643
(@ite _ p h q (decide p)) = (decide p && q) := by
644644
split <;> simp_all
645645

646-
@[deprecated ite_then_decide_self]
646+
@[deprecated ite_then_decide_self (since := "2024-08-29")]
647647
theorem ite_true_decide_same (p : Prop) [Decidable p] (b : Bool) :
648648
(if p then decide p else b) = (decide p || b) := ite_then_decide_self p b
649649

650-
@[deprecated ite_false_decide_same]
650+
@[deprecated ite_false_decide_same (since := "2024-08-29")]
651651
theorem ite_false_decide_same (p : Prop) [Decidable p] (b : Bool) :
652652
(if p then b else decide p) = (decide p && b) := ite_else_decide_self p b
653653

src/Lean/Data/HashMap.lean

Lines changed: 6 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -271,11 +271,11 @@ def ofListWith (l : List (α × β)) (f : β → β → β) : HashMap α β :=
271271
| none => m.insert p.fst p.snd
272272
| some v => m.insert p.fst $ f v p.snd)
273273

274-
attribute [deprecated Std.HashMap] HashMap
275-
attribute [deprecated Std.HashMap.Raw] HashMapImp
276-
attribute [deprecated Std.HashMap.Raw.empty] mkHashMapImp
277-
attribute [deprecated Std.HashMap.empty] mkHashMap
278-
attribute [deprecated Std.HashMap.empty] HashMap.empty
279-
attribute [deprecated Std.HashMap.ofList] HashMap.ofList
274+
attribute [deprecated Std.HashMap (since := "2024-08-08")] HashMap
275+
attribute [deprecated Std.HashMap.Raw (since := "2024-08-08")] HashMapImp
276+
attribute [deprecated Std.HashMap.Raw.empty (since := "2024-08-08")] mkHashMapImp
277+
attribute [deprecated Std.HashMap.empty (since := "2024-08-08")] mkHashMap
278+
attribute [deprecated Std.HashMap.empty (since := "2024-08-08")] HashMap.empty
279+
attribute [deprecated Std.HashMap.ofList (since := "2024-08-08")] HashMap.ofList
280280

281281
end Lean.HashMap

src/Lean/Data/HashSet.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -219,8 +219,8 @@ def merge {α : Type u} [BEq α] [Hashable α] (s t : HashSet α) : HashSet α :
219219
t.fold (init := s) fun s a => s.insert a
220220
-- We don't use `insertMany` here because it gives weird universes.
221221

222-
attribute [deprecated Std.HashSet] HashSet
223-
attribute [deprecated Std.HashSet.Raw] HashSetImp
224-
attribute [deprecated Std.HashSet.Raw.empty] mkHashSetImp
225-
attribute [deprecated Std.HashSet.empty] mkHashSet
226-
attribute [deprecated Std.HashSet.empty] HashSet.empty
222+
attribute [deprecated Std.HashSet (since := "2024-08-08")] HashSet
223+
attribute [deprecated Std.HashSet.Raw (since := "2024-08-08")] HashSetImp
224+
attribute [deprecated Std.HashSet.Raw.empty (since := "2024-08-08")] mkHashSetImp
225+
attribute [deprecated Std.HashSet.empty (since := "2024-08-08")] mkHashSet
226+
attribute [deprecated Std.HashSet.empty (since := "2024-08-08")] HashSet.empty

src/Lean/Meta/Tactic/Apply.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -254,7 +254,7 @@ Apply `And.intro` as much as possible to goal `mvarId`.
254254
abbrev splitAnd (mvarId : MVarId) : MetaM (List MVarId) :=
255255
splitAndCore mvarId
256256

257-
@[deprecated splitAnd] -- 2024-03-17
257+
@[deprecated splitAnd (since := "2024-03-17")]
258258
def _root_.Lean.Meta.splitAnd (mvarId : MVarId) : MetaM (List MVarId) :=
259259
mvarId.splitAnd
260260

src/Std/Data/HashMap/Basic.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -118,7 +118,7 @@ Tries to retrieve the mapping for the given key, returning `none` if no such map
118118
@[inline] def get? (m : HashMap α β) (a : α) : Option β :=
119119
DHashMap.Const.get? m.inner a
120120

121-
@[deprecated get? "Use `m[a]?` or `m.get? a` instead", inherit_doc get?]
121+
@[deprecated get? "Use `m[a]?` or `m.get? a` instead" (since := "2024-08-07"), inherit_doc get?]
122122
def find? (m : HashMap α β) (a : α) : Option β :=
123123
m.get? a
124124

@@ -145,7 +145,7 @@ Retrieves the mapping for the given key. Ensures that such a mapping exists by r
145145
(fallback : β) : β :=
146146
DHashMap.Const.getD m.inner a fallback
147147

148-
@[deprecated getD, inherit_doc getD]
148+
@[deprecated getD (since := "2024-08-07"), inherit_doc getD]
149149
def findD (m : HashMap α β) (a : α) (fallback : β) : β :=
150150
m.getD a fallback
151151

@@ -157,7 +157,7 @@ Tries to retrieve the mapping for the given key, panicking if no such mapping is
157157
@[inline] def get! [Inhabited β] (m : HashMap α β) (a : α) : β :=
158158
DHashMap.Const.get! m.inner a
159159

160-
@[deprecated get! "Use `m[a]!` or `m.get! a` instead", inherit_doc get!]
160+
@[deprecated get! "Use `m[a]!` or `m.get! a` instead" (since := "2024-08-07"), inherit_doc get!]
161161
def find! [Inhabited β] (m : HashMap α β) (a : α) : Option β :=
162162
m.get! a
163163

0 commit comments

Comments
 (0)