Documentation

Mathlib.Topology.Algebra.InfiniteSum.ENNReal

Infinite sums of ENNReal and Set.encard #

This file provides lemmas relating sums of constants to the cardinality of the domain of these sums.

TODO #

@[simp]
theorem ENNReal.tsum_set_one_eq {α : Type u_1} (s : Set α) :
∑' (x : s), 1 = s.encard
@[simp]
theorem ENNReal.tsum_set_const_eq {α : Type u_1} (s : Set α) (c : ENNReal) :
∑' (x : s), c = s.encard * c