Zulip Chat Archive
Stream: Is there code for X?
Topic: Triangular infinite sums
Eric Wieser (Jan 06 2024 at 11:14):
Do we have anything along the lines of:
/-- An infinite triangular sum can be transposed. -/
theorem HasSum_sum_range_iff {α} [TopologicalSpace α] [AddCommMonoid α] [ContinuousAdd α]
(f : ℕ → ℕ → α) (a : α):
HasSum (fun n => ∑ k in .range n, f n k) a ↔ HasSum (fun nk : ℕ × ℕ => f (nk.1 + nk.2) nk.2) a :=
sorry
That is, that ? (modulo off-by-one errors)
Antoine Chambert-Loir (Jan 07 2024 at 16:02):
That's a particular case of Fubini, and it wouldn't bet that it holds without an additional absolute summability assumption.
Last updated: May 02 2025 at 03:31 UTC