Skip to content

Commit

Permalink
lemma
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Nov 6, 2024
1 parent 66ac702 commit 39258ab
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/Lean/SimpLC/Whitelists/List.lean
Original file line number Diff line number Diff line change
Expand Up @@ -91,6 +91,12 @@ simp_lc ignore List.foldl_subtype
simp_lc ignore List.foldr_subtype
simp_lc ignore List.mapFinIdx_eq_mapIdx

-- TODO move to library.
@[simp] theorem List.modifyHead_dropLast {l : List α} : l.dropLast.modifyHead f = (l.modifyHead f).dropLast:= by
rcases l with _|⟨a, l⟩
· simp
· rcases l with _|⟨b, l⟩ <;> simp

/-
The actual checks happen in `tests/lean/run/simplc.lean`.
This commented out command remains here for convenience while debugging.
Expand Down

0 comments on commit 39258ab

Please sign in to comment.