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 derivative 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.iteratedFDerivβ': wrapsiteratedFDerivinto aπ-linear map onContDiffMapSupportedIn E F n K, as a map intoContDiffMapSupportedIn E (E [Γi]βL[β] F) (n-i) K.
Main statements #
TODO:
ContDiffMapSupportedIn.instIsUniformAddGroupandContDiffMapSupportedIn.instLocallyConvexSpace:ContDiffMapSupportedInis a locally convex topological vector space.
Notation #
π^{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).
Implementation details #
The technical choice of spelling EqOn f 0 KαΆ in the definition, as opposed to tsupport f β K
is to make rewriting f x to 0 easier when x β K.
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 (inifinitely 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
continously 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' := β― }