Skip to content

Commit 2c97fe4

Browse files
committed
lemma
1 parent fe60957 commit 2c97fe4

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

src/Lean/SimpLC/Whitelists/List.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -91,6 +91,12 @@ simp_lc ignore List.foldl_subtype
9191
simp_lc ignore List.foldr_subtype
9292
simp_lc ignore List.mapFinIdx_eq_mapIdx
9393

94+
-- TODO move to library.
95+
@[simp] theorem List.modifyHead_dropLast {l : List α} : l.dropLast.modifyHead f = (l.modifyHead f).dropLast:= by
96+
rcases l with _|⟨a, l⟩
97+
· simp
98+
· rcases l with _|⟨b, l⟩ <;> simp
99+
94100
/-
95101
The actual checks happen in `tests/lean/run/simplc.lean`.
96102
This commented out command remains here for convenience while debugging.

0 commit comments

Comments
 (0)