Skip to content

Commit

Permalink
Update Std/Data/List/Lemmas.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Kim Morrison <kim@tqft.net>
  • Loading branch information
tjf801 and semorrison committed May 1, 2024
1 parent 61ba0bd commit 2b57fb6
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Std/Data/List/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -365,7 +365,7 @@ theorem exists_of_mem_join : a ∈ join L → ∃ l, l ∈ L ∧ a ∈ l := mem_

theorem mem_join_of_mem (lL : l ∈ L) (al : a ∈ l) : a ∈ join L := mem_join.2 ⟨l, lL, al⟩

theorem length_join (l : List (List α)) : (join l).length = Nat.sum (l.map length) := by
theorem length_join (l : List (List α)) : (join l).length = (l.map length).sum := by
induction l <;> simp [*]

/-! ### bind -/
Expand Down

0 comments on commit 2b57fb6

Please sign in to comment.