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 8b0815e commit 2ea88b1Copy full SHA for 2ea88b1
Mathlib/Data/List/Basic.lean
@@ -509,9 +509,6 @@ theorem get_cons {l : List α} {a : α} {n} (hl) :
509
l.get ⟨n - 1, by contrapose! hl; rw [length_cons]; omega⟩ :=
510
getElem_cons hl
511
512
-theorem modifyHead_modifyHead (l : List α) (f g : α → α) :
513
- (l.modifyHead f).modifyHead g = l.modifyHead (g ∘ f) := by cases l <;> simp
514
-
515
/-! ### Induction from the right -/
516
517
/-- Induction principle from the right for lists: if a property holds for the empty list, and
0 commit comments