Zulip Chat Archive
Stream: Is there code for X?
Topic: finsupp equals sum of `finsupp.filter`
Andrew Yang (Oct 15 2022 at 18:40):
Is there a good way to prove the lemma below?
import data.finsupp.basic
example {α β γ : Type*} [add_comm_monoid β] (f : α → γ) (x : α →₀ β) {P : (α →₀ β) → Prop}
  (h₁ : ∀ b, P (x.filter (λ a, f a = b)))
  (h₂ : ∀ x y, P x → P y → P (x + y)) : P x :=
begin
end
Andrew Yang (Oct 15 2022 at 19:23):
I managed to state and proof the statement in the title :
lemma finsupp.sum_image_support_filter {α β γ : Type*}
  [add_comm_monoid β] (f : α → γ) (x : α →₀ β) [decidable_eq γ] :
  ∑ b in finset.image f x.support, x.filter (λ a, f a = b) = x :=
begin
  ext i,
  simp_rw [finsupp.finset_sum_apply, finsupp.filter_apply, finset.sum_ite, finset.sum_const_zero,
    add_zero, finset.filter_eq],
  split_ifs,
  { simp },
  { rw [finset.sum_empty, eq_comm, ← finsupp.not_mem_support_iff],
    exact λ h', h (finset.mem_image_of_mem f h') }
end
Is this not in mathlib? Is there any generalizations?
Last updated: May 02 2025 at 03:31 UTC