Documentation

Mathlib.MeasureTheory.Integral.RieszMarkovKakutani.Real

Riesz–Markov–Kakutani representation theorem for real-linear functionals #

The Riesz–Markov–Kakutani representation theorem relates linear functionals on spaces of continuous functions on a locally compact space to measures.

There are many closely related variations of the theorem. This file contains that proof of the version where the space is a locally compact T2 space, the linear functionals are real and the continuous functions have compact support.

Main definitions & statements #

Implementation notes #

The measure is defined through rieszContent which is for NNReal using the toNNRealLinear version of Λ.

The Riesz–Markov–Kakutani representation theorem is first proved for Real-linear Λ because equality is proven using two inequalities by considering Λ f and Λ (-f) for all functions f, yet on C_c(X, ℝ≥0) there is no negation.

References #

The measure induced for Real-linear positive functional Λ, defined through toNNRealLinear and the NNReal-version of rieszContent. This is under the namespace RealRMK, while rieszMeasure without namespace is for NNReal-linear Λ.

Equations
Instances For

    If f assumes values between 0 and 1 and the support is contained in V, then Λ f ≤ rieszMeasure V.

    theorem RealRMK.rieszMeasure_le_of_eq_one {X : Type u_1} [TopologicalSpace X] [T2Space X] [LocallyCompactSpace X] [MeasurableSpace X] [BorelSpace X] {Λ : CompactlySupportedContinuousMap X →ₗ[] } ( : ∀ (f : CompactlySupportedContinuousMap X ), 0 f0 Λ f) {f : CompactlySupportedContinuousMap X } (hf : ∀ (x : X), 0 f x) {K : Set X} (hK : IsCompact K) (hfK : xK, f x = 1) :

    If f assumes the value 1 on a compact set K then rieszMeasure K ≤ Λ f.

    theorem RealRMK.range_cut_partition {X : Type u_1} [TopologicalSpace X] [MeasurableSpace X] [BorelSpace X] (f : CompactlySupportedContinuousMap X ) (a : ) {ε : } ( : 0 < ε) (N : ) (hf : Set.range f Set.Ioo a (a + N * ε)) :
    ∃ (E : Fin NSet X), tsupport f = ⋃ (j : Fin N), E j Set.univ.PairwiseDisjoint E (∀ (n : Fin N), xE n, a + ε * n < f x f x a + ε * (n + 1)) ∀ (n : Fin N), MeasurableSet (E n)

    Given f : C_c(X, ℝ) such that range f ⊆ [a, b] we obtain a partition of the support of f determined by partitioning [a, b] into N pieces.

    theorem RealRMK.exists_open_approx {X : Type u_1} [TopologicalSpace X] [T2Space X] [MeasurableSpace X] [BorelSpace X] (f : CompactlySupportedContinuousMap X ) {ε : } ( : 0 < ε) (E : Set X) {μ : MeasureTheory.Content X} ( : μ.outerMeasure E ) (hμ' : MeasurableSet E) {c : } (hfE : xE, f x < c) :
    ∃ (V : TopologicalSpace.Opens X), E V (∀ xV, f x < c) μ.measure V μ.measure E + ENNReal.ofReal ε

    Given a set E, a function f : C_c(X, ℝ), 0 < ε and ∀ x ∈ E, f x < c, there exists an open set V such that E ⊆ V and the sets are similar in measure and ∀ x ∈ V, f x < c.

    The Riesz-Markov-Kakutani representation theorem: given a positive linear functional Λ, the integral of f with respect to the rieszMeasure associated to Λ is equal to Λ f.