Documentation

Mathlib.Analysis.Calculus.BumpFunction.FiniteDimension

Bump functions in finite-dimensional vector spaces #

Let E be a finite-dimensional real normed vector space. We show that any open set s in E is exactly the support of a smooth function taking values in [0, 1], in IsOpen.exists_smooth_support_eq.

Then we use this construction to construct bump functions with nice behavior, by convolving the indicator function of closedBall 0 1 with a function as above with s = ball 0 D.

theorem exists_smooth_tsupport_subset {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] {s : Set E} {x : E} (hs : s nhds x) :

If a set s is a neighborhood of x, then there exists a smooth function f taking values in [0, 1], supported in s and with f x = 1.

Given an open set s in a finite-dimensional real normed vector space, there exists a smooth function with values in [0, 1] whose support is exactly s.

An auxiliary function to construct partitions of unity on finite-dimensional real vector spaces. It is the characteristic function of the closed unit ball.

Equations
Instances For
    theorem ExistsContDiffBumpBase.u_exists (E : Type u_1) [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] :
    ∃ (u : E), ContDiff u (∀ (x : E), u x Set.Icc 0 1) Function.support u = Metric.ball 0 1 ∀ (x : E), u (-x) = u x

    An auxiliary function to construct partitions of unity on finite-dimensional real vector spaces, which is smooth, symmetric, and with support equal to the unit ball.

    Equations
    Instances For
      theorem ExistsContDiffBumpBase.u_int_pos (E : Type u_1) [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [MeasurableSpace E] [BorelSpace E] :
      0 < ∫ (x : E), ExistsContDiffBumpBase.u xMeasureTheory.Measure.addHaar

      An auxiliary function to construct partitions of unity on finite-dimensional real vector spaces, which is smooth, symmetric, with support equal to the ball of radius D and integral 1.

      Equations
      Instances For
        theorem ExistsContDiffBumpBase.w_integral (E : Type u_1) [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [MeasurableSpace E] [BorelSpace E] {D : } (Dpos : 0 < D) :
        ∫ (x : E), ExistsContDiffBumpBase.w D xMeasureTheory.Measure.addHaar = 1

        An auxiliary function to construct partitions of unity on finite-dimensional real vector spaces. It is the convolution between a smooth function of integral 1 supported in the ball of radius D, with the indicator function of the closed unit ball. Therefore, it is smooth, equal to 1 on the ball of radius 1 - D, with support equal to the ball of radius 1 + D.

        Equations
        Instances For
          theorem ExistsContDiffBumpBase.y_pos_of_mem_ball {E : Type u_1} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [MeasurableSpace E] [BorelSpace E] {D : } {x : E} (Dpos : 0 < D) (D_lt_one : D < 1) (hx : x Metric.ball 0 (1 + D)) :