Documentation

Mathlib.Topology.ContinuousMap.BoundedCompactlySupported

Compactly supported bounded continuous functions #

The two-sided ideal of compactly supported bounded continuous functions taking values in a metric space, with the uniform distance.

The two-sided ideal of compactly supported functions.

Equations
    Instances For

      The two-sided ideal of compactly supported functions.

      Equations
        Instances For
          theorem exist_norm_eq {α : Type u_1} {γ : Type u_2} [TopologicalSpace α] [NonUnitalNormedRing γ] [c : Nonempty α] {f : BoundedContinuousFunction α γ} (h : f compactlySupported α γ) :
          ∃ (x : α), f x = f
          theorem norm_lt_iff_of_compactlySupported {α : Type u_1} {γ : Type u_2} [TopologicalSpace α] [NonUnitalNormedRing γ] {f : BoundedContinuousFunction α γ} (h : f compactlySupported α γ) {M : } (M0 : 0 < M) :
          f < M ∀ (x : α), f x < M
          theorem norm_lt_iff_of_nonempty_compactlySupported {α : Type u_1} {γ : Type u_2} [TopologicalSpace α] [NonUnitalNormedRing γ] [c : Nonempty α] {f : BoundedContinuousFunction α γ} (h : f compactlySupported α γ) {M : } :
          f < M ∀ (x : α), f x < M
          def ofCompactSupport {α : Type u_1} {γ : Type u_2} [TopologicalSpace α] [NonUnitalNormedRing γ] (g : αγ) (hg₁ : Continuous g) (hg₂ : HasCompactSupport g) :

          A compactly supported continuous function is automatically bounded. This constructor gives an object of α →ᵇ γ from g : α → γ and these assumptions.

          Equations
            Instances For
              theorem ofCompactSupport_mem {α : Type u_1} {γ : Type u_2} [TopologicalSpace α] [NonUnitalNormedRing γ] (g : αγ) (hg₁ : Continuous g) (hg₂ : HasCompactSupport g) :