Skip to content

Commit cc241e9

Browse files
committed
deprecations
1 parent 16cdffe commit cc241e9

File tree

5 files changed

+6
-6
lines changed

5 files changed

+6
-6
lines changed

Batteries/Control/AlternativeMonad.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -104,7 +104,7 @@ section AlternativeMonad
104104

105105
@[simp] theorem seq_failure [AlternativeMonad m] [LawfulAlternative m] [LawfulMonad m]
106106
(x : m (α → β)) : x <*> failure = x *> failure := by
107-
simp only [seq_eq_bind, map_failure, seqRight_eq, bind_map_left]
107+
simp only [seq_eq_bind_map, map_failure, seqRight_eq, bind_map_left]
108108

109109
end AlternativeMonad
110110

Batteries/Data/Array/Match.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -58,7 +58,7 @@ def PrefixTable.extend [BEq α] (t : PrefixTable α) (x : α) : PrefixTable α w
5858
rw [Array.getElem_push]
5959
split
6060
· exact t.valid ..
61-
· next h => exact Nat.le_trans (Nat.lt_succ.1 <| Fin.isLt ..) (Nat.not_lt.1 h)
61+
· next h => exact Nat.le_trans (Nat.lt_succ_iff.1 <| Fin.isLt ..) (Nat.not_lt.1 h)
6262

6363
/-- Make prefix table from a pattern array -/
6464
def mkPrefixTable [BEq α] (xs : Array α) : PrefixTable α := xs.foldl (·.extend) default

Batteries/Data/UnionFind/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -145,7 +145,7 @@ theorem rank'_lt_rankMax (self : UnionFind) (i : Nat) (h) : (self.arr[i]).rank <
145145
| a::l, _, List.Mem.head _ => by dsimp; apply Nat.le_max_left
146146
| a::l, _, .tail _ h => by dsimp; exact Nat.le_trans (go h) (Nat.le_max_right ..)
147147
simp only [rankMax, ← Array.foldr_toList]
148-
exact Nat.lt_succ.2 <| go (self.arr.toList.getElem_mem _)
148+
exact Nat.lt_succ_iff.2 <| go (self.arr.toList.getElem_mem _)
149149

150150
theorem rankD_lt_rankMax (self : UnionFind) (i : Nat) :
151151
rankD self.arr i < self.rankMax := by

Batteries/Data/UnionFind/Lemmas.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -22,7 +22,7 @@ namespace Batteries.UnionFind
2222
parentD (arr.push ⟨arr.size, 0⟩) a = parentD arr a := by
2323
simp [parentD]; split <;> split <;> try simp [Array.getElem_push, *]
2424
· next h1 h2 =>
25-
simp [Nat.lt_succ] at h1 h2
25+
simp [Nat.lt_succ_iff] at h1 h2
2626
exact Nat.le_antisymm h2 h1
2727
· next h1 h2 => cases h1 (Nat.lt_succ_of_lt h2)
2828

Batteries/Lean/EStateM.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -70,14 +70,14 @@ theorem run_seq (f : EStateM ε σ (α → β)) (x : EStateM ε σ α) (s : σ)
7070
(f <*> x).run s = match f.run s with
7171
| .ok g s => Result.map g (x.run s)
7272
| .error e s => .error e s := by
73-
simp only [seq_eq_bind, run_bind, run_map]
73+
simp only [seq_eq_bind_map, run_bind, run_map]
7474
cases f.run s <;> rfl
7575

7676
theorem run'_seq (f : EStateM ε σ (α → β)) (x : EStateM ε σ α) (s : σ) :
7777
(f <*> x).run' s = match f.run s with
7878
| .ok g s => Option.map g (x.run' s)
7979
| .error _ _ => none := by
80-
simp only [seq_eq_bind, run'_bind, run'_map]
80+
simp only [seq_eq_bind_map, run'_bind, run'_map]
8181
cases f.run s <;> rfl
8282

8383
@[simp] theorem run_seqLeft (x : EStateM ε σ α) (y : EStateM ε σ β) (s : σ) :

0 commit comments

Comments
 (0)