Skip to content

Commit d5a05a3

Browse files
committed
fix
1 parent 18a408b commit d5a05a3

File tree

1 file changed

+0
-4
lines changed

1 file changed

+0
-4
lines changed

src/Init/Data/Array/Lemmas.lean

Lines changed: 0 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -239,10 +239,6 @@ theorem back?_pop {xs : Array α} :
239239

240240
@[simp] theorem push_empty : #[].push x = #[x] := rfl
241241

242-
@[simp] theorem toList_push {xs : Array α} {x : α} : (xs.push x).toList = xs.toList ++ [x] := by
243-
rcases xs with ⟨xs⟩
244-
simp
245-
246242
@[simp] theorem push_ne_empty {a : α} {xs : Array α} : xs.push a ≠ #[] := by
247243
cases xs
248244
simp

0 commit comments

Comments
 (0)