Documentation

Mathlib.MeasureTheory.Function.ContinuousMapDense

Approximation in Lᵖ by continuous functions #

This file proves that bounded continuous functions are dense in Lp E p μ, for p < ∞, if the domain α of the functions is a normal topological space and the measure μ is weakly regular. It also proves the same results for approximation by continuous functions with compact support when the space is locally compact and μ is regular.

The result is presented in several versions. First concrete versions giving an approximation up to ε in these various contexts, and then abstract versions stating that the topological closure of the relevant subgroups of Lp are the whole space.

Versions with Integrable instead of Memℒp are specialized to the case p = 1. Versions with boundedContinuous instead of HasCompactSupport drop the locally compact assumption and give only approximation by a bounded continuous function.

Note that for p = ∞ this result is not true: the characteristic function of the set [0, ∞) in cannot be continuously approximated in L∞.

The proof is in three steps. First, since simple functions are dense in Lp, it suffices to prove the result for a scalar multiple of a characteristic function of a measurable set s. Secondly, since the measure μ is weakly regular, the set s can be approximated above by an open set and below by a closed set. Finally, since the domain α is normal, we use Urysohn's lemma to find a continuous function interpolating between these two sets.

Are you looking for a result on "directional" approximation (above or below with respect to an order) of functions whose codomain is ℝ≥0∞ or , by semicontinuous functions? See the Vitali-Carathéodory theorem, in the file Mathlib/MeasureTheory/Integral/VitaliCaratheodory.lean.

theorem MeasureTheory.exists_continuous_snorm_sub_le_of_closed {α : Type u_1} [MeasurableSpace α] [TopologicalSpace α] [T4Space α] [BorelSpace α] {E : Type u_2} [NormedAddCommGroup E] {μ : MeasureTheory.Measure α} {p : ENNReal} [NormedSpace E] [MeasureTheory.Measure.OuterRegular μ] (hp : p ) {s : Set α} {u : Set α} (s_closed : IsClosed s) (u_open : IsOpen u) (hsu : s u) (hs : μ s ) (c : E) {ε : ENNReal} (hε : ε 0) :
∃ (f : αE), Continuous f MeasureTheory.snorm (fun (x : α) => f x - Set.indicator s (fun (_y : α) => c) x) p μ ε (∀ (x : α), f x c) Function.support f u MeasureTheory.Memℒp f p μ

A variant of Urysohn's lemma, ℒ^p version, for an outer regular measure μ: consider two sets s ⊆ u which are respectively closed and open with μ s < ∞, and a vector c. Then one may find a continuous function f equal to c on s and to 0 outside of u, bounded by ‖c‖ everywhere, and such that the ℒ^p norm of f - s.indicator (fun y ↦ c) is arbitrarily small. Additionally, this function f belongs to ℒ^p.

In a locally compact space, any function in ℒp can be approximated by compactly supported continuous functions when p < ∞, version in terms of snorm.

theorem MeasureTheory.Memℒp.exists_hasCompactSupport_integral_rpow_sub_le {α : Type u_1} [MeasurableSpace α] [TopologicalSpace α] [T4Space α] [BorelSpace α] {E : Type u_2} [NormedAddCommGroup E] {μ : MeasureTheory.Measure α} [NormedSpace E] [WeaklyLocallyCompactSpace α] [MeasureTheory.Measure.Regular μ] {p : } (hp : 0 < p) {f : αE} (hf : MeasureTheory.Memℒp f (ENNReal.ofReal p) μ) {ε : } (hε : 0 < ε) :
∃ (g : αE), HasCompactSupport g ∫ (x : α), f x - g x ^ pμ ε Continuous g MeasureTheory.Memℒp g (ENNReal.ofReal p) μ

In a locally compact space, any function in ℒp can be approximated by compactly supported continuous functions when 0 < p < ∞, version in terms of .

In a locally compact space, any integrable function can be approximated by compactly supported continuous functions, version in terms of ∫⁻.

In a locally compact space, any integrable function can be approximated by compactly supported continuous functions, version in terms of .

Any function in ℒp can be approximated by bounded continuous functions when p < ∞, version in terms of snorm.

theorem MeasureTheory.Memℒp.exists_boundedContinuous_integral_rpow_sub_le {α : Type u_1} [MeasurableSpace α] [TopologicalSpace α] [T4Space α] [BorelSpace α] {E : Type u_2} [NormedAddCommGroup E] {μ : MeasureTheory.Measure α} [NormedSpace E] [MeasureTheory.Measure.WeaklyRegular μ] {p : } (hp : 0 < p) {f : αE} (hf : MeasureTheory.Memℒp f (ENNReal.ofReal p) μ) {ε : } (hε : 0 < ε) :
∃ (g : BoundedContinuousFunction α E), ∫ (x : α), f x - g x ^ pμ ε MeasureTheory.Memℒp (g) (ENNReal.ofReal p) μ

Any function in ℒp can be approximated by bounded continuous functions when 0 < p < ∞, version in terms of .

Any integrable function can be approximated by bounded continuous functions, version in terms of ∫⁻.

Any integrable function can be approximated by bounded continuous functions, version in terms of .

Continuous functions are dense in MeasureTheory.Lp, 1 ≤ p < ∞. This theorem assumes that the domain is a compact space because otherwise ContinuousMap.toLp is undefined. Use BoundedContinuousFunction.toLp_denseRange if the domain is not a compact space.