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 ebf455a commit a8cf5feCopy full SHA for a8cf5fe
src/Init/Data/List/TakeDrop.lean
@@ -31,6 +31,11 @@ theorem take_cons {l : List α} (h : 0 < i) : (a :: l).take i = a :: l.take (i -
31
| zero => exact absurd h (Nat.lt_irrefl _)
32
| succ i => rfl
33
34
+theorem drop_cons {l : List α} (h : 0 < i) : (a :: l).drop i = l.drop (i - 1) := by
35
+ cases i with
36
+ | zero => exact absurd h (Nat.lt_irrefl _)
37
+ | succ i => rfl
38
+
39
@[simp]
40
theorem drop_one : ∀ {l : List α}, l.drop 1 = l.tail
41
| [] | _ :: _ => rfl
0 commit comments