Skip to content

Commit

Permalink
Update Lemmas.lean
Browse files Browse the repository at this point in the history
  • Loading branch information
eric-wieser authored Nov 18, 2024
1 parent 7a0b786 commit 8943fce
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Data/List/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2395,7 +2395,7 @@ theorem forall_mem_replicate {p : α → Prop} {a : α} {n} :

@[simp] theorem getElem_replicate (a : α) {n : Nat} {m} (h : m < (replicate n a).length) :
(replicate n a)[m] = a :=
eq_of_mem_replicate (get_mem _ _ _)
eq_of_mem_replicate (getElem_mem _)

@[deprecated getElem_replicate (since := "2024-06-12")]
theorem get_replicate (a : α) {n : Nat} (m : Fin _) : (replicate n a).get m = a := by
Expand Down

0 comments on commit 8943fce

Please sign in to comment.