Zulip Chat Archive
Stream: new members
Topic: A question about ENNReal
Ching-Tsun Chou (Dec 15 2024 at 00:41):
Under the assumption that:
variable (ι : Type*) (s : Set ι) (h : s.Infinite) (c : ENNReal)
how does one go about proving that the following sum:
∑' (_ : ↑s), c
is either 0 or infinity depending on whether c is 0 or positive?
Matt Diamond (Dec 15 2024 at 00:53):
docs#ENNReal.tsum_const_eq_top_of_ne_zero should be useful here (along with docs#tsum_zero)
Matt Diamond (Dec 15 2024 at 01:08):
import Mathlib
variable (ι : Type*) (s : Set ι) (h : s.Infinite) (c : ENNReal)
example (hc : c = 0) : ∑' (_ : ↑s), c = 0 := by rw [hc, tsum_zero]
example (hc : c ≠ 0) : ∑' (_ : ↑s), c = ⊤ :=
have : Infinite ↑s := h.to_subtype
ENNReal.tsum_const_eq_top_of_ne_zero hc
Ching-Tsun Chou (Dec 15 2024 at 03:49):
Thanks! That's exactly what I need.
Last updated: May 02 2025 at 03:31 UTC