Skip to content

Commit

Permalink
feat: List.map_id' with lambda (#450)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Dec 15, 2023
1 parent 75e75a5 commit fa17cba
Showing 1 changed file with 2 additions and 0 deletions.
2 changes: 2 additions & 0 deletions Std/Data/List/Init/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -103,6 +103,8 @@ theorem append_left_inj {s₁ s₂ : List α} (t) : s₁ ++ t = s₂ ++ t ↔ s

@[simp] theorem map_id (l : List α) : map id l = l := by induction l <;> simp_all

@[simp] theorem map_id' (l : List α) : map (fun a => a) l = l := by induction l <;> simp_all

@[simp] theorem map_map (g : β → γ) (f : α → β) (l : List α) :
map g (map f l) = map (g ∘ f) l := by induction l <;> simp_all

Expand Down

0 comments on commit fa17cba

Please sign in to comment.