Infinite sum and products that converge uniformly #
Main definitions #
HasProdUniformlyOn f g s:∏ i, f i bconverges uniformly onstog.HasProdLocallyUniformlyOn f g s:∏ i, f i bconverges locally uniformly onstog.HasProdUniformly f g:∏ i, f i bconverges uniformly tog.HasProdLocallyUniformly f g:∏ i, f i bconverges locally uniformly tog.
Uniform convergence of sums and products #
HasProdUniformlyOn f g s means that the (potentially infinite) product ∏' i, f i b
for b : β converges uniformly on s to g.
Equations
- HasProdUniformlyOn f g s = HasProd (⇑(UniformOnFun.ofFun {s}) ∘ f) ((UniformOnFun.ofFun {s}) g)
Instances For
HasSumUniformlyOn f g s means that the (potentially infinite) sum ∑' i, f i b
for b : β converges uniformly on s to g.
Equations
- HasSumUniformlyOn f g s = HasSum (⇑(UniformOnFun.ofFun {s}) ∘ f) ((UniformOnFun.ofFun {s}) g)
Instances For
MultipliableUniformlyOn f s means that there is some infinite product to which
f converges uniformly on s. Use fun x ↦ ∏' i, f i x to get the product function.
Equations
- MultipliableUniformlyOn f s = Multipliable (⇑(UniformOnFun.ofFun {s}) ∘ f)
Instances For
SummableUniformlyOn f s means that there is some infinite sum to
which f converges uniformly on s. Use fun x ↦ ∑' i, f i x to get the sum function.
Equations
- SummableUniformlyOn f s = Summable (⇑(UniformOnFun.ofFun {s}) ∘ f)
Instances For
Alias of the forward direction of hasProdUniformlyOn_iff_tendstoUniformlyOn.
Alias of HasProdUniformlyOn.tprod_eqOn.
Alias of HasSumUniformlyOn.tsum_eqOn.
Locally uniform convergence of sums and products #
HasProdLocallyUniformlyOn f g s means that the (potentially infinite) product ∏' i, f i b
for b : β converges locally uniformly on s to g b (in the sense of
TendstoLocallyUniformlyOn).
Equations
- HasProdLocallyUniformlyOn f g s = TendstoLocallyUniformlyOn (fun (x1 : Finset ι) (x2 : β) => ∏ i ∈ x1, f i x2) g Filter.atTop s
Instances For
HasSumLocallyUniformlyOn f g s means that the (potentially infinite) sum
∑' i, f i b for b : β converges locally uniformly on s to g b (in the sense of
TendstoLocallyUniformlyOn).
Equations
- HasSumLocallyUniformlyOn f g s = TendstoLocallyUniformlyOn (fun (x1 : Finset ι) (x2 : β) => ∑ i ∈ x1, f i x2) g Filter.atTop s
Instances For
MultipliableLocallyUniformlyOn f s means that the product ∏' i, f i b converges locally
uniformly on s to something.
Equations
- MultipliableLocallyUniformlyOn f s = ∃ (g : β → α), HasProdLocallyUniformlyOn f g s
Instances For
SummableLocallyUniformlyOn f s means that ∑' i, f i b converges locally
uniformly on s to something.
Equations
- SummableLocallyUniformlyOn f s = ∃ (g : β → α), HasSumLocallyUniformlyOn f g s
Instances For
If every x ∈ s has a neighbourhood within s on which b ↦ ∏' i, f i b converges uniformly
to g, then the product converges locally uniformly on s to g. Note that this is not a
tautology, and the converse is only true if the domain is locally compact.
If every x ∈ s has a neighbourhood within s on which b ↦ ∑' i, f i b
converges uniformly to g, then the sum converges locally uniformly. Note that this is not a
tautology, and the converse is only true if the domain is locally compact.
Alias of hasProdLocallyUniformlyOn_of_of_forall_exists_nhds.
If every x ∈ s has a neighbourhood within s on which b ↦ ∏' i, f i b converges uniformly
to g, then the product converges locally uniformly on s to g. Note that this is not a
tautology, and the converse is only true if the domain is locally compact.
Alias of hasSumLocallyUniformlyOn_of_of_forall_exists_nhds.
If every x ∈ s has a neighbourhood within s on which b ↦ ∑' i, f i b
converges uniformly to g, then the sum converges locally uniformly. Note that this is not a
tautology, and the converse is only true if the domain is locally compact.
If every x ∈ s has a neighbourhood within s on which b ↦ ∏' i, f i b converges uniformly,
then the product converges locally uniformly on s. Note that this is not a tautology, and the
converse is only true if the domain is locally compact.
If every x ∈ s has a neighbourhood within s on which b ↦ ∑' i, f i b
converges uniformly, then the sum converges locally uniformly. Note that this is not a tautology,
and the converse is only true if the domain is locally compact.
Alias of multipliableLocallyUniformlyOn_of_of_forall_exists_nhds.
If every x ∈ s has a neighbourhood within s on which b ↦ ∏' i, f i b converges uniformly,
then the product converges locally uniformly on s. Note that this is not a tautology, and the
converse is only true if the domain is locally compact.
Alias of summableLocallyUniformlyOn_of_of_forall_exists_nhds.
If every x ∈ s has a neighbourhood within s on which b ↦ ∑' i, f i b
converges uniformly, then the sum converges locally uniformly. Note that this is not a tautology,
and the converse is only true if the domain is locally compact.
HasProdUniformly f g means that
the product ∏ i, f i b converges uniformly (wrt b) to g.
Equations
- HasProdUniformly f g = HasProd (⇑UniformFun.ofFun ∘ f) (UniformFun.ofFun g)
Instances For
HasSumUniformly f g means that
the sum ∑ i, f i b converges uniformly (wrt b) to g.
Equations
- HasSumUniformly f g = HasSum (⇑UniformFun.ofFun ∘ f) (UniformFun.ofFun g)
Instances For
MultipliableUniformly f means that there is some infinite product to which
f converges uniformly. Use fun x ↦ ∏' i, f i x to get the product function.
Equations
Instances For
SummableUniformly f means that there is some infinite sum to which
f converges uniformly. Use fun x ↦ ∑' i, f i x to get the product function.
Equations
- SummableUniformly f = Summable (⇑UniformFun.ofFun ∘ f)
Instances For
Alias of the forward direction of hasProdUniformly_iff_tendstoUniformly.
Locally uniform convergence of sums and products #
HasProdLocallyUniformly f g means that the (potentially infinite) product ∏' i, f i b
for b : β converges locally uniformly to g b (in the sense of
TendstoLocallyUniformly).
Equations
- HasProdLocallyUniformly f g = TendstoLocallyUniformly (fun (x1 : Finset ι) (x2 : β) => ∏ i ∈ x1, f i x2) g Filter.atTop
Instances For
HasSumLocallyUniformly f g means that the (potentially infinite) sum
∑' i, f i b for b : β converges locally uniformly to g b (in the sense of
TendstoLocallyUniformly).
Equations
- HasSumLocallyUniformly f g = TendstoLocallyUniformly (fun (x1 : Finset ι) (x2 : β) => ∑ i ∈ x1, f i x2) g Filter.atTop
Instances For
MultipliableLocallyUniformly f means that the product ∏' i, f i b converges locally
uniformly to something.
Equations
- MultipliableLocallyUniformly f = ∃ (g : β → α), HasProdLocallyUniformly f g
Instances For
SummableLocallyUniformly f means that ∑' i, f i b converges locally
uniformly to something.
Equations
- SummableLocallyUniformly f = ∃ (g : β → α), HasSumLocallyUniformly f g
Instances For
If every x has a neighbourhood on which b ↦ ∏' i, f i b converges uniformly
to g, then the product converges locally uniformly to g. Note that this is not a
tautology, and the converse is only true if the domain is locally compact.
If every x has a neighbourhood on which b ↦ ∑' i, f i b
converges uniformly to g, then the sum converges locally uniformly. Note that this is not a
tautology, and the converse is only true if the domain is locally compact.