Infinite sum in a ring #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file provides lemmas about the interaction between infinite sums and multiplication.
Main results #
tsum_mul_tsum_eq_tsum_sum_antidiagonal
: Cauchy product formula
Multipliying two infinite sums #
In this section, we prove various results about (∑' x : ι, f x) * (∑' y : κ, g y)
. Note that we
always assume that the family λ x : ι × κ, f x.1 * g x.2
is summable, since there is no way to
deduce this from the summmabilities of f
and g
in general, but if you are working in a normed
space, you may want to use the analogous lemmas in analysis/normed_space/basic
(e.g tsum_mul_tsum_of_summable_norm
).
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
).
Arbitrary index types #
Product of two infinites sums indexed by arbitrary types.
See also tsum_mul_tsum_of_summable_norm
if f
and g
are abolutely 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
, 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
,
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 infinites sums indexed by ℕ
, expressed
by summing on finset.nat.antidiagonal
.
See also tsum_mul_tsum_eq_tsum_sum_antidiagonal_of_summable_norm
if f
and g
are absolutely
summable.
The Cauchy product formula for the product of two infinites sums indexed by ℕ
, expressed
by summing on finset.range
.
See also tsum_mul_tsum_eq_tsum_sum_range_of_summable_norm
if f
and g
are absolutely summable.