Skip to content

Commit

Permalink
Update Std/Data/String/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 2b57fb6 commit c96137c
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Std/Data/String/Lemmas.lean
Original file line number Diff line number Diff line change
Expand Up @@ -501,7 +501,7 @@ theorem join_eq (ss : List String) : join ss = ⟨(ss.map data).join⟩ := go ss

@[simp] theorem comp_length_data : List.length ∘ String.data = String.length := rfl

theorem length_join (l : List String) : (String.join l).length = Nat.sum (l.map String.length) := by
theorem length_join (l : List String) : (String.join l).length = (l.map String.length).sum := by
simp [length, List.length_join, List.map_map]

theorem singleton_eq (c : Char) : singleton c = ⟨[c]⟩ := rfl
Expand Down

0 comments on commit c96137c

Please sign in to comment.