We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 18a408b commit d5a05a3Copy full SHA for d5a05a3
src/Init/Data/Array/Lemmas.lean
@@ -239,10 +239,6 @@ theorem back?_pop {xs : Array α} :
239
240
@[simp] theorem push_empty : #[].push x = #[x] := rfl
241
242
-@[simp] theorem toList_push {xs : Array α} {x : α} : (xs.push x).toList = xs.toList ++ [x] := by
243
- rcases xs with ⟨xs⟩
244
- simp
245
-
246
@[simp] theorem push_ne_empty {a : α} {xs : Array α} : xs.push a ≠ #[] := by
247
cases xs
248
simp
0 commit comments