Skip to content

Commit

Permalink
Update Mathlib/Algebra/FreeMonoid/Count.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Ruben Van de Velde <[email protected]>
  • Loading branch information
edegeltje and Ruben-VandeVelde authored Jan 22, 2025
1 parent 1895dc6 commit 36eb824
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/FreeMonoid/Count.lean
Original file line number Diff line number Diff line change
Expand Up @@ -44,7 +44,7 @@ theorem countP_apply (l : FreeMonoid α) : l.countP p = .ofAdd (l.toList.countP
lemma countP_of (x : α) : (of x).countP p =
if p x then Multiplicative.ofAdd 1 else Multiplicative.ofAdd 0 := by
rw [countP_apply, toList_of, List.countP_singleton, apply_ite (Multiplicative.ofAdd)]
simp only [decide_eq_true_eq, ofAdd_zero]
simp only [decide_eq_true_eq]


/-- `List.count` as a bundled additive monoid homomorphism. -/
Expand Down

0 comments on commit 36eb824

Please sign in to comment.