Infinite sum and product in a topological monoid #
This file defines infinite products and sums for (possibly infinite) indexed families of elements in a commutative topological monoid (resp. add monoid).
To handle convergence questions we use the formalism of summation filters (defined in the
file Mathlib.Topology.Algebra.InfiniteSum.SummationFilter
). These are filters on the finite
subsets of a given type, and we define a function to be summable for a summation filter L
if
its partial sums over finite subsets tend to a limit along L
(and similarly for products).
This simultaneously generalizes several different kinds of summation: for instance,
unconditional summation (which makes sense for any index type) where we take the limit with
respect to the atTop
filter; but also conditional summation for functions on ℕ
, where the
limit is over the partial sums ∑ i ∈ range n, f i
as n → ∞
(so there exist
conditionally-summable sequences which are not unconditionally summable).
Implementation notes #
We say that a function f : β → α
has a product of a
w.r.t. the summation filter L
if the
function fun s : Finset β ↦ ∏ b ∈ s, f b
converges to a
w.r.t. the filter L.filter
on
Finset β
.
In the most important case of unconditional summation, this translates to the following condition:
for every neighborhood U
of a
, there exists a finite set s : Finset β
of indices such
that ∏ b ∈ s', f b ∈ U
for any finite set s'
which is a superset of s
.
This may yield some unexpected results. For example, according to this definition, the product
∏' n : ℕ, (1 : ℝ) / 2
unconditionally exists and is equal to 0
. More strikingly,
the product ∏' n : ℕ, (n : ℝ)
unconditionally exists and is equal to 0
, because one
of its terms is 0
(even though the product of the remaining terms diverges). Users who would
prefer that these products be considered not to exist can carry them out in the unit group ℝˣ
rather than in ℝ
.
References #
- Bourbaki: General Topology (1995), Chapter 3 §5 (Infinite sums in commutative groups)
HasProd f a L
means that the (potentially infinite) product of the f b
for b : β
converges
to a
along the SummationFilter L
.
By default L
is the unconditional
one, corresponding to the limit of all finite sets towards
the entire type. So we take the product over bigger and bigger finite sets. This product operation
is invariant under permuting the terms (while products for more general summation filters usually
are not).
For the definition and many statements, α
does not need to be a topological monoid, only a monoid
with a topology (i.e. the multiplication is not assumed to be continuous). We only add this
assumption later, for the lemmas where it is relevant.
These are defined in an identical way to infinite sums (HasSum
). For example, we say that
the function ℕ → ℝ
sending n
to 1 / 2
has a product of 0
, rather than saying that it does
not converge as some authors would.
Instances For
HasSum f a L
means that the (potentially infinite) sum of the f b
for b : β
converges to a
along the SummationFilter `L``.
By default L
is the unconditional
one, corresponding to the limit of all finite sets towards
the entire type. So we take the sum over bigger and bigger finite sets. This sum operation is
invariant under permuting the terms (while sums for more general summation filters usually are not).
This is based on Mario Carneiro's
infinite sum df-tsms
in Metamath.
In particular, the function ℕ → ℝ
sending n
to (-1) ^ n / (n + 1)
does not have a
sum for this definition, although it is summable for the conditional
summation filter that
takes limits of sums over n ∈ {0, ..., X}
as X → ∞
. However, a series which is absolutely
convergent with respect to the conditional summation filter is in fact unconditionally summable.
For the definition and many statements, α
does not need to be a topological additive monoid,
only an additive monoid with a topology (i.e. the addition is not assumed to be continuous). We
only add this assumption later, for the lemmas where it is relevant.
Instances For
Multipliable f
means that f
has some (infinite) product with respect to L
. Use tprod
to
get the value.
Equations
- Multipliable f L = ∃ (a : α), HasProd f a L
Instances For
Summable f
means that f
has some (infinite) sum with respect to L
. Use tsum
to get the
value.
Instances For
∏' i, f i
is the unconditional product of f
, if it exists, or 1 otherwise. ]
More generally, if L
is a SummationFilter
, ∏'[L] i, f i
is the product of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional product exists, it might not be unique if the topology is not
separated. When the multiplicative support of f
is finite, we make the most reasonable choice,
to use the product over the multiplicative support. Otherwise, we choose arbitrarily an a
satisfying HasProd f a
. Similar remarks apply to more general summation filters.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
∑' i, f i
is the unconditional sum of f
if it exists, or 0 otherwise.
More generally, if L
is a SummationFilter
, ∑'[L] i, f i
is the sum of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional sum exists, it might not be unique if the topology is not
separated. When the support of f
is finite, we make the most reasonable choice, to use the sum
over the support. Otherwise, we choose arbitrarily an a
satisfying HasSum f a
. Similar remarks
apply to more general summation filters.)
Equations
Instances For
∑' i, f i
is the unconditional sum of f
if it exists, or 0 otherwise.
More generally, if L
is a SummationFilter
, ∑'[L] i, f i
is the sum of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional sum exists, it might not be unique if the topology is not
separated. When the support of f
is finite, we make the most reasonable choice, to use the sum
over the support. Otherwise, we choose arbitrarily an a
satisfying HasSum f a
. Similar remarks
apply to more general summation filters.)
∏' i, f i
is the unconditional product of f
, if it exists, or 1 otherwise. ]
More generally, if L
is a SummationFilter
, ∏'[L] i, f i
is the product of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional product exists, it might not be unique if the topology is not
separated. When the multiplicative support of f
is finite, we make the most reasonable choice,
to use the product over the multiplicative support. Otherwise, we choose arbitrarily an a
satisfying HasProd f a
. Similar remarks apply to more general summation filters.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
∑' i, f i
is the unconditional sum of f
if it exists, or 0 otherwise.
More generally, if L
is a SummationFilter
, ∑'[L] i, f i
is the sum of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional sum exists, it might not be unique if the topology is not
separated. When the support of f
is finite, we make the most reasonable choice, to use the sum
over the support. Otherwise, we choose arbitrarily an a
satisfying HasSum f a
. Similar remarks
apply to more general summation filters.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
∏' i, f i
is the unconditional product of f
, if it exists, or 1 otherwise. ]
More generally, if L
is a SummationFilter
, ∏'[L] i, f i
is the product of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional product exists, it might not be unique if the topology is not
separated. When the multiplicative support of f
is finite, we make the most reasonable choice,
to use the product over the multiplicative support. Otherwise, we choose arbitrarily an a
satisfying HasProd f a
. Similar remarks apply to more general summation filters.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
∑' i, f i
is the unconditional sum of f
if it exists, or 0 otherwise.
More generally, if L
is a SummationFilter
, ∑'[L] i, f i
is the sum of f
with respect to
L
if it exists, and 1
otherwise.
(Note that even if the unconditional sum exists, it might not be unique if the topology is not
separated. When the support of f
is finite, we make the most reasonable choice, to use the sum
over the support. Otherwise, we choose arbitrarily an a
satisfying HasSum f a
. Similar remarks
apply to more general summation filters.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
If the summation filter is the trivial filter ⊥
, then the topological product is equal to the
finite product (which is taken to be 1 if the multiplicative support of f
is infinite).
Note that in this case HasProd f a
is satisfied for every element a
of the target, so the
value assigned to the tprod
is a question of conventions.
If the summation filter is the trivial filter ⊥
, then the topological sum is
equal to the finite sum (which is taken to be 1 if the support of f
is infinite).
Note that in this case HasSum f a
is satisfied for every element a
of the target, so the
value assigned to the tsum
is a question of conventions.
If a function f
is 1
outside of a finite set s
, then it HasProd
∏ b ∈ s, f b
.
If a function f
vanishes outside of a finite set s
, then it HasSum
∑ b ∈ s, f b
.
If a function f
is 1
outside of a finite set s
, then it HasProd
∏ b ∈ s, f b
.
If a function f
vanishes outside of a finite set s
, then it HasSum
∑ b ∈ s, f b
.