Skip to content

Commit e65df5a

Browse files
committed
spaces
1 parent 670b397 commit e65df5a

File tree

8 files changed

+11
-11
lines changed

8 files changed

+11
-11
lines changed

src/Init/Data/Array/Lemmas.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -2798,7 +2798,7 @@ theorem reverse_eq_iff {xs ys : Array α} : xs.reverse = ys ↔ xs = ys.reverse
27982798
cases xs
27992799
simp
28002800

2801-
@[grind _=_]theorem filterMap_reverse {f : α → Option β} {xs : Array α} : (xs.reverse.filterMap f) = (xs.filterMap f).reverse := by
2801+
@[grind _=_] theorem filterMap_reverse {f : α → Option β} {xs : Array α} : (xs.reverse.filterMap f) = (xs.filterMap f).reverse := by
28022802
cases xs
28032803
simp
28042804

@@ -3527,7 +3527,7 @@ theorem foldrM_append [Monad m] [LawfulMonad m] {f : α → β → m β} {b} {xs
35273527
(xs ++ ys).foldr f b start 0 = xs.foldr f (ys.foldr f b) :=
35283528
foldrM_append' w
35293529

3530-
@[grind _=_]theorem foldl_append {β : Type _} {f : β → α → β} {b} {xs ys : Array α} :
3530+
@[grind _=_] theorem foldl_append {β : Type _} {f : β → α → β} {b} {xs ys : Array α} :
35313531
(xs ++ ys).foldl f b = ys.foldl f (xs.foldl f b) :=
35323532
foldlM_append
35333533

src/Init/Data/List/Nat/TakeDrop.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -56,7 +56,7 @@ theorem getElem?_take_eq_none {l : List α} {i j : Nat} (h : i ≤ j) :
5656
(l.take i)[j]? = none :=
5757
getElem?_eq_none <| Nat.le_trans (length_take_le _ _) h
5858

59-
@[grind =]theorem getElem?_take {l : List α} {i j : Nat} :
59+
@[grind =] theorem getElem?_take {l : List α} {i j : Nat} :
6060
(l.take i)[j]? = if j < i then l[j]? else none := by
6161
split
6262
· next h => exact getElem?_take_of_lt h

src/Init/Data/Vector/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2105,7 +2105,7 @@ abbrev forall_mem_mkVector := @forall_mem_replicate
21052105
@[deprecated getElem_replicate (since := "2025-03-18")]
21062106
abbrev getElem_mkVector := @getElem_replicate
21072107

2108-
@[grind]theorem getElem?_replicate {a : α} {n i : Nat} : (replicate n a)[i]? = if i < n then some a else none := by
2108+
@[grind] theorem getElem?_replicate {a : α} {n i : Nat} : (replicate n a)[i]? = if i < n then some a else none := by
21092109
simp [getElem?_def]
21102110

21112111
@[deprecated getElem?_replicate (since := "2025-03-18")]

src/Std/Data/DTreeMap/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3961,7 +3961,7 @@ theorem getKey?_maxKey! [TransCmp cmp] [Inhabited α] (he : t.isEmpty = false) :
39613961
t.getKey? t.maxKey! = some t.maxKey! :=
39623962
Impl.getKey?_maxKey! t.wf he
39633963

3964-
@[grind =]theorem getKey_maxKey! [TransCmp cmp] [Inhabited α] {hc} :
3964+
@[grind =] theorem getKey_maxKey! [TransCmp cmp] [Inhabited α] {hc} :
39653965
t.getKey t.maxKey! hc = t.maxKey! :=
39663966
Impl.getKey_maxKey! t.wf
39673967

src/Std/Data/ExtDHashMap/Lemmas.lean

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -305,7 +305,7 @@ theorem get_eq_get_get? [LawfulBEq α] {a : α} {h} :
305305
m.get a h = (m.get? a).get (mem_iff_isSome_get?.mp h) :=
306306
m.inductionOn (fun _ _ => DHashMap.get_eq_get_get?) h
307307

308-
@[grind =]theorem get_get? [LawfulBEq α] {a : α} {h} :
308+
@[grind =] theorem get_get? [LawfulBEq α] {a : α} {h} :
309309
(m.get? a).get h = m.get a (mem_iff_isSome_get?.mpr h) :=
310310
m.inductionOn (fun _ _ => DHashMap.get_get?) h
311311

@@ -405,7 +405,7 @@ variable {β : Type v} {m : ExtDHashMap α (fun _ => β)}
405405
theorem get!_empty [EquivBEq α] [LawfulHashable α] [Inhabited β] {a : α} : get! (∅ : ExtDHashMap α (fun _ => β)) a = default :=
406406
DHashMap.Const.get!_empty
407407

408-
@[grind =]theorem get!_insert [EquivBEq α] [LawfulHashable α] [Inhabited β] {k a : α} {v : β} :
408+
@[grind =] theorem get!_insert [EquivBEq α] [LawfulHashable α] [Inhabited β] {k a : α} {v : β} :
409409
get! (m.insert k v) a = if k == a then v else get! m a :=
410410
m.inductionOn fun _ => DHashMap.Const.get!_insert
411411

@@ -462,7 +462,7 @@ theorem getD_empty [LawfulBEq α] {a : α} {fallback : β a} :
462462
(∅ : ExtDHashMap α β).getD a fallback = fallback :=
463463
DHashMap.getD_empty
464464

465-
@[grind =]theorem getD_insert [LawfulBEq α] {k a : α} {fallback : β a} {v : β k} :
465+
@[grind =] theorem getD_insert [LawfulBEq α] {k a : α} {fallback : β a} {v : β k} :
466466
(m.insert k v).getD a fallback =
467467
if h : k == a then cast (congrArg β (eq_of_beq h)) v else m.getD a fallback :=
468468
m.inductionOn fun _ => DHashMap.getD_insert

src/Std/Data/HashSet/RawLemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -167,7 +167,7 @@ theorem contains_insert_self [EquivBEq α] [LawfulHashable α] (h : m.WF) {k :
167167
theorem mem_insert_self [EquivBEq α] [LawfulHashable α] (h : m.WF) {k : α} : k ∈ m.insert k :=
168168
HashMap.Raw.mem_insertIfNew_self h.out
169169

170-
@[grind =]theorem size_insert [EquivBEq α] [LawfulHashable α] (h : m.WF) {k : α} :
170+
@[grind =] theorem size_insert [EquivBEq α] [LawfulHashable α] (h : m.WF) {k : α} :
171171
(m.insert k).size = if k ∈ m then m.size else m.size + 1 :=
172172
HashMap.Raw.size_insertIfNew h.out
173173

src/Std/Data/TreeMap/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -2001,7 +2001,7 @@ theorem minKey?_modify_eq_minKey? [TransCmp cmp] [LawfulEqCmp cmp] {k f} :
20012001
(t.modify k f).minKey? = t.minKey? :=
20022002
DTreeMap.Const.minKey?_modify_eq_minKey?
20032003

2004-
@[grind =]theorem isSome_minKey?_modify [TransCmp cmp] {k f} :
2004+
@[grind =] theorem isSome_minKey?_modify [TransCmp cmp] {k f} :
20052005
(t.modify k f).minKey?.isSome = !t.isEmpty :=
20062006
DTreeMap.Const.isSome_minKey?_modify
20072007

src/Std/Data/TreeSet/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -347,7 +347,7 @@ theorem getD_of_isEmpty [TransCmp cmp] {a fallback : α} :
347347
t.isEmpty = true → t.getD a fallback = fallback :=
348348
TreeMap.getKeyD_of_isEmpty
349349

350-
@[grind =]theorem getD_insert [TransCmp cmp] {k a fallback : α} :
350+
@[grind =] theorem getD_insert [TransCmp cmp] {k a fallback : α} :
351351
(t.insert k).getD a fallback =
352352
if cmp k a = .eq ∧ ¬ k ∈ t then k else t.getD a fallback :=
353353
TreeMap.getKeyD_insertIfNew

0 commit comments

Comments
 (0)