Skip to content

Commit 2401996

Browse files
committed
deprecations
1 parent d5a05a3 commit 2401996

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/Init/Data/Array/Attach.lean

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -69,11 +69,11 @@ well-founded recursion mechanism to prove that the function terminates.
6969
simp [pmap]
7070

7171
@[simp] theorem toList_attachWith {xs : Array α} {P : α → Prop} {H : ∀ x ∈ xs, P x} :
72-
(xs.attachWith P H).toList = xs.toList.attachWith P (by simpa [mem_toList] using H) := by
72+
(xs.attachWith P H).toList = xs.toList.attachWith P (by simpa [mem_toList_iff] using H) := by
7373
simp [attachWith]
7474

7575
@[simp] theorem toList_attach {xs : Array α} :
76-
xs.attach.toList = xs.toList.attachWith (· ∈ xs) (by simp [mem_toList]) := by
76+
xs.attach.toList = xs.toList.attachWith (· ∈ xs) (by simp [mem_toList_iff]) := by
7777
simp [attach]
7878

7979
@[simp] theorem toList_pmap {xs : Array α} {P : α → Prop} {f : ∀ a, P a → β} {H : ∀ a ∈ xs, P a} :

src/Init/Data/Array/Zip.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -373,7 +373,7 @@ theorem unzip_zip {as : Array α} {bs : Array β} (h : as.size = bs.size) :
373373

374374
theorem zip_of_prod {as : Array α} {bs : Array β} {xs : Array (α × β)} (hl : xs.map Prod.fst = as)
375375
(hr : xs.map Prod.snd = bs) : xs = as.zip bs := by
376-
rw [← hl, ← hr, ← zip_unzip xs, ← unzip_fst, ← unzip_snd, zip_unzip, zip_unzip]
376+
rw [← hl, ← hr, ← zip_unzip xs, ← fst_unzip, ← snd_unzip, zip_unzip, zip_unzip]
377377

378378
@[simp] theorem unzip_replicate {n : Nat} {a : α} {b : β} :
379379
unzip (replicate n (a, b)) = (replicate n a, replicate n b) := by

0 commit comments

Comments
 (0)