Documentation

Mathlib.Analysis.Distribution.ContDiffMapSupportedIn

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:

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 #

Main statements #

TODO:

Notation #

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.

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
        class ContDiffMapSupportedInClass (B : Type u_4) (E : outParam (Type u_5)) (F : outParam (Type u_6)) [NormedAddCommGroup E] [NormedAddCommGroup F] [NormedSpace ℝ E] [NormedSpace ℝ F] (n : outParam β„•βˆž) (K : outParam (TopologicalSpace.Compacts E)) extends DFunLike B E fun (x : E) => F :
        Type (max (max u_4 u_5) u_6)

        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.

        Instances
          Equations

          See note [custom simps projection].

          Equations
          Instances For
            theorem ContDiffMapSupportedIn.ext {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ℝ E] [NormedAddCommGroup F] [NormedSpace ℝ F] {n : β„•βˆž} {K : TopologicalSpace.Compacts E} {f g : ContDiffMapSupportedIn E F n K} (h : βˆ€ (a : E), f a = g a) :
            f = g
            def ContDiffMapSupportedIn.copy {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ℝ E] [NormedAddCommGroup F] [NormedSpace ℝ F] {n : β„•βˆž} {K : TopologicalSpace.Compacts E} (f : ContDiffMapSupportedIn E F n K) (f' : E β†’ F) (h : f' = ⇑f) :

            Copy of a ContDiffMapSupportedIn with a new toFun equal to the old one. Useful to fix definitional equalities.

            Equations
            • f.copy f' h = { toFun := f', contDiff' := β‹―, zero_on_compl' := β‹― }
            Instances For
              @[simp]
              theorem ContDiffMapSupportedIn.coe_copy {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ℝ E] [NormedAddCommGroup F] [NormedSpace ℝ F] {n : β„•βˆž} {K : TopologicalSpace.Compacts E} (f : ContDiffMapSupportedIn E F n K) (f' : E β†’ F) (h : f' = ⇑f) :
              ⇑(f.copy f' h) = f'
              theorem ContDiffMapSupportedIn.copy_eq {E : Type u_2} {F : Type u_3} [NormedAddCommGroup E] [NormedSpace ℝ E] [NormedAddCommGroup F] [NormedSpace ℝ F] {n : β„•βˆž} {K : TopologicalSpace.Compacts E} (f : ContDiffMapSupportedIn E F n K) (f' : E β†’ F) (h : f' = ⇑f) :
              f.copy f' h = f