Continuously differentiable functions supported in a given compact set #
This file develops the basic theory of bundled n-times continuously differentiable functions
with support contained in a given compact set.
Given n : ββ and a compact subset K of a normed space E, we consider the type of bundled
functions f : E β F (where F is a normed vector space) such that:
fisn-times continuously differentiable:ContDiff β n f.fvanishes outside of a compact set:EqOn f 0 KαΆ.
The main reason this exists as a bundled type is to be endowed with its natural locally convex
topology (namely, uniform convergence of f and its derivatives up to order n).
Taking the locally convex inductive limit of these as K varies yields the natural topology on test
functions, used to define distributions. While most of distribution theory cares only about C^β
functions, we also want to endow the space of C^n test functions with its natural topology.
Indeed, distributions of order less than n are precisely those which extend continuously to this
larger space of test functions.
Main definitions #
ContDiffMapSupportedIn E F n K: the type of bundledn-times continuously differentiable functionsE β Fwhich vanish outside ofK.ContDiffMapSupportedIn.iteratedFDerivWithOrderLM: wrapper, as aπ-linear map, foriteratedFDerivfromContDiffMapSupportedIn E F n KtoContDiffMapSupportedIn E (E [Γi]βL[β] F) k K.ContDiffMapSupportedIn.iteratedFDerivLM: specialization of the above, giving aπ-linear map fromContDiffMapSupportedIn E F β€ KtoContDiffMapSupportedIn E (E [Γi]βL[β] F) β€ K.ContDiffMapSupportedIn.topologicalSpace,ContDiffMapSupportedIn.uniformSpace: the topology and uniform structures onπ^{n}_{K}(E, F), given by uniform convergence of the functions and all their derivatives up to ordern.
Main statements #
ContDiffMapSupportedIn.isTopologicalAddGroup,ContDiffMapSupportedIn.continuousSMulandContDiffMapSupportedIn.instLocallyConvexSpace:π^{n}_{K}(E, F)is a locally convex topological vector space.
Notation #
In the Distributions scope, we introduce the following notations:
π^{n}_{K}(E, F): the space ofn-times continuously differentiable functionsE β Fwhich vanish outside ofK.π_{K}(E, F): the space of smooth (infinitely differentiable) functionsE β Fwhich vanish outside ofK, i.e.π^{β€}_{K}(E, F).N[π; F]_{K, n, i}(or simplyN[π]_{K, n, i}): theπ-seminorm onπ^{n}_{K}(E, F)given by the sup-norm of thei-th derivative.N[π; F]_{K, i}(or simplyN[π]_{K, i}): theπ-seminorm onπ_{K}(E, F)given by the sup-norm of thei-th derivative.
Implementation details #
- The technical choice of spelling
EqOn f 0 KαΆin the definition, as opposed totsupport f β Kis to make rewritingf xto0easier whenx β K. - Since the most common case is by far the smooth case, we often reserve the "expected" name
of a result/definition to this case, and add
WithOrderto the declaration applying to any regularity. - In
iteratedFDerivWithOrderLM, we define thei-th iterated differentiation operator as a map fromπ^{n}_{K}toπ^{k}_{K}without imposing relations onn,kandi. Of course this is defined as0ifk + i > n. This creates some verbosity as all of these variables are explicit, but it allows the most flexibility while avoiding DTT hell.
Tags #
distributions
The type of bundled n-times continuously differentiable maps which vanish outside of a fixed
compact set K.
- toFun : E β F
The underlying function. Use coercion instead.
Instances For
Notation for the space of bundled n-times continuously differentiable
functions with support in a compact set K.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Notation for the space of bundled smooth (infinitely differentiable)
functions with support in a compact set K.
Equations
- One or more equations did not get rendered due to their size.
Instances For
ContDiffMapSupportedInClass B E F n K states that B is a type of bundled n-times
continuously differentiable functions with support in the compact set K.
- coe : B β (a : E) β F
Instances
Equations
- ContDiffMapSupportedIn.toContDiffMapSupportedInClass E F = { coe := fun (f : ContDiffMapSupportedIn E F n K) => f.toFun, coe_injective' := β―, map_contDiff := β―, map_zero_on_compl := β― }
See note [custom simps projection].
Equations
Instances For
Copy of a ContDiffMapSupportedIn with a new toFun equal to the old one. Useful to fix
definitional equalities.
Instances For
Equations
- ContDiffMapSupportedIn.instAdd = { add := fun (f g : ContDiffMapSupportedIn E F n K) => { toFun := βf + βg, contDiff' := β―, zero_on_compl' := β― } }
Equations
- ContDiffMapSupportedIn.instNeg = { neg := fun (f : ContDiffMapSupportedIn E F n K) => { toFun := -βf, contDiff' := β―, zero_on_compl' := β― } }
Equations
- ContDiffMapSupportedIn.instSub = { sub := fun (f g : ContDiffMapSupportedIn E F n K) => { toFun := βf - βg, contDiff' := β―, zero_on_compl' := β― } }
Equations
- ContDiffMapSupportedIn.instSMul = { smul := fun (c : R) (f : ContDiffMapSupportedIn E F n K) => { toFun := c β’ βf, contDiff' := β―, zero_on_compl' := β― } }
Equations
- One or more equations did not get rendered due to their size.
Coercion as an additive homomorphism.
Equations
- ContDiffMapSupportedIn.coeHom E F n K = { toFun := fun (f : ContDiffMapSupportedIn E F n K) => βf, map_zero' := β―, map_add' := β― }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Inclusion of unbundled n-times continuously differentiable function with support included
in a compact K into the space π^{n}_{K}.
Equations
- ContDiffMapSupportedIn.of_support_subset hf hsupp = { toFun := f, contDiff' := hf, zero_on_compl' := β― }
Instances For
Inclusion of π^{n}_{K}(E, F) into the space E βα΅ F of bounded continuous maps
as a π-linear map.
This is subsumed by toBoundedContinuousFunctionCLM, which also bundles the continuity.
Equations
- One or more equations did not get rendered due to their size.
Instances For
iteratedFDerivWithOrderLM π n k i is the π-linear-map sending f : π^{n}_{K}(E, F) to
its i-th iterated derivative as an element of π^{k}_{K}(E, E [Γi]βL[β] F).
This only makes mathematical sense if k + i β€ n, otherwise we define it as the zero map.
See iteratedFDerivLM for the very common case where everything is infinitely differentiable.
This is subsumed by iteratedFDerivWithOrderCLM (not yet in Mathlib), which also bundles the
continuity.
Equations
- One or more equations did not get rendered due to their size.
Instances For
iteratedFDerivLM π i is the π-linear-map sending f : π_{K}(E, F) to
its i-th iterated derivative as an element of π_{K}(E, E [Γi]βL[β] F).
See also iteratedFDerivWithOrderLM if you need more control on the regularities.
This is subsumed by iteratedFDerivCLM (not yet in Mathlib), which also bundles the
continuity.
Equations
- ContDiffMapSupportedIn.iteratedFDerivLM π i = { toFun := fun (f : ContDiffMapSupportedIn E F β€ K) => ContDiffMapSupportedIn.of_support_subset β― β―, map_add' := β―, map_smul' := β― }
Instances For
Note: this turns out to be a definitional equality thanks to decidablity of the order
on ββ. This means we could have defined iteratedFDerivLM this way, but we avoid it
to make sure that ifs won't appear in the smooth case.
structureMapLM π n i is the π-linear-map sending f : π^{n}_{K}(E, F) to its
i-th iterated derivative as an element of E βα΅ (E [Γi]βL[β] F). In other words, it
is the composition of toBoundedContinuousFunctionLM π and iteratedFDerivWithOrderLM π n 0 i.
This only makes mathematical sense if i β€ n, otherwise we define it as the zero map.
We call these "structure maps" because they define the topology on π^{n}_{K}(E, F).
This is subsumed by structureMapCLM, which also bundles the
continuity.
Equations
Instances For
Equations
Equations
- ContDiffMapSupportedIn.uniformSpace = (β¨ (i : β), UniformSpace.comap (β(ContDiffMapSupportedIn.structureMapLM β n i)) inferInstance).replaceTopology β―
structureMapCLM π n i is the continuous π-linear-map sending f : π^{n}_{K}(E, F) to its
i-th iterated derivative as an element of E βα΅ (E [Γi]βL[β] F).
This only makes mathematical sense if i β€ n, otherwise we define it as the zero map.
We call these "structure maps" because they define the topology on π^{n}_{K}(E, F).
Equations
- ContDiffMapSupportedIn.structureMapCLM π n i = { toLinearMap := ContDiffMapSupportedIn.structureMapLM π n i, cont := β― }
Instances For
The universal property of the topology on π^{n}_{K}(E, F): a map to π^{n}_{K}(E, F)
is continuous if and only if its composition with each structure map
structureMapCLM β n i : π^{n}_{K}(E, F) β (E βα΅ (E [Γi]βL[β] F)) is continuous.
Since structureMapCLM β n i is zero whenever i > n, it suffices to check it for i β€ n,
as proven by continuous_iff_comp_withOrder.
The universal property of the topology on π^{n}_{K}(E, F): a map to π^{n}_{K}(E, F)
is continuous if and only if its composition with the structure map
structureMapCLM β n i : π^{n}_{K}(E, F) β (E βα΅ (E [Γi]βL[β] F)) is continuous for each
i β€ n.
The seminorms on the space π^{n}_{K}(E, F) given by the sup norm of the iterated derivatives.
In the scope Distributions.Seminorm, we denote them by N[π; F]_{K, n, i}
(or N[π]_{K, n, i}), or simply by N[π; F]_{K, i} (or N[π; F]_{K, i}) when n = β.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The seminorms on the space π^{n}_{K}(E, F) given by the sup norm of the iterated derivatives.
In the scope Distributions.Seminorm, we denote them by N[π; F]_{K, n, i}
(or N[π]_{K, n, i}), or simply by N[π; F]_{K, i} (or N[π; F]_{K, i}) when n = β.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The seminorms on the space π^{n}_{K}(E, F) given by the sup norm of the iterated derivatives.
In the scope Distributions.Seminorm, we denote them by N[π; F]_{K, n, i}
(or N[π]_{K, n, i}), or simply by N[π; F]_{K, i} (or N[π; F]_{K, i}) when n = β.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The seminorms on the space π^{n}_{K}(E, F) given by the sup norm of the iterated derivatives.
In the scope Distributions.Seminorm, we denote them by N[π; F]_{K, n, i}
(or N[π]_{K, n, i}), or simply by N[π; F]_{K, i} (or N[π; F]_{K, i}) when n = β.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The seminorms on the space π^{n}_{K}(E, F) given by the sup norm of the iterated derivatives.
In the scope Distributions.Seminorm, we denote them by N[π; F]_{K, n, i}
(or N[π]_{K, n, i}), or simply by N[π; F]_{K, i} (or N[π; F]_{K, i}) when n = β.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The seminorms on the space π^{n}_{K}(E, F) given by sup of the
ContDiffMapSupportedIn.seminorm kfor k β€ i.
Equations
- ContDiffMapSupportedIn.supSeminorm π E F n K i = (Finset.Iic i).sup (ContDiffMapSupportedIn.seminorm π E F n K)
Instances For
The inclusion of the space π^{n}_{K}(E, F) into the space E βα΅ F of bounded continuous
functions as a continuous π-linear map.
Equations
- ContDiffMapSupportedIn.toBoundedContinuousFunctionCLM π = { toLinearMap := ContDiffMapSupportedIn.toBoundedContinuousFunctionLM π, cont := β― }