Documentation

Mathlib.Algebra.BigOperators.Ring.Nat

Big operators on a finset in the natural numbers #

This file contains the results concerning the interaction of finset big operators with natural numbers.

theorem Finset.even_sum_iff_even_card_odd {ι : Type u_1} {s : Finset ι} (f : ι) :
Even (∑ is, f i) Even {xs | Odd (f x)}.card
theorem Finset.odd_sum_iff_odd_card_odd {ι : Type u_1} {s : Finset ι} (f : ι) :
Odd (∑ is, f i) Odd {xs | Odd (f x)}.card
theorem Finset.card_preimage_eq_sum_card_image_eq {ι : Type u_1} {M : Type u_2} {f : ιM} {s : Finset M} (hb : bs, {a : ι | f a = b}.Finite) :
Nat.card ↑(f ⁻¹' s) = bs, Nat.card { a : ι // f a = b }