Multiplying two infinite sums in a normed ring #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file, we prove various results about (∑' x : ι, f x) * (∑' y : ι', g y) in a normed
ring. There are similar results proven in topology/algebra/infinite_sum (e.g tsum_mul_tsum),
but in a normed ring we get summability results which aren't true in general.
We first establish results about arbitrary index types, β and γ, and then we specialize to
β = γ = ℕ to prove the Cauchy product formula
(see tsum_mul_tsum_eq_tsum_sum_antidiagonal_of_summable_norm).
!
Arbitrary index types #
Product of two infinites sums indexed by arbitrary types.
See also tsum_mul_tsum if f and g are not absolutely summable.
ℕ-indexed families (Cauchy product) #
We prove two versions of the Cauchy product formula. The first one is
tsum_mul_tsum_eq_tsum_sum_range_of_summable_norm, where the n-th term is a sum over
finset.range (n+1) involving nat subtraction.
In order to avoid nat subtraction, we also provide
tsum_mul_tsum_eq_tsum_sum_antidiagonal_of_summable_norm,
where the n-th term is a sum over all pairs (k, l) such that k+l=n, which corresponds to the
finset finset.nat.antidiagonal n.
The Cauchy product formula for the product of two infinite sums indexed by ℕ,
expressed by summing on finset.nat.antidiagonal.
See also tsum_mul_tsum_eq_tsum_sum_antidiagonal if f and g are
not absolutely summable.
The Cauchy product formula for the product of two infinite sums indexed by ℕ,
expressed by summing on finset.range.
See also tsum_mul_tsum_eq_tsum_sum_range if f and g are
not absolutely summable.