Documentation

Mathlib.MeasureTheory.Measure.Lebesgue.Basic

Lebesgue measure on the real line and on ℝⁿ #

We show that the Lebesgue measure on the real line (constructed as a particular case of additive Haar measure on inner product spaces) coincides with the Stieltjes measure associated to the function x ↦ x. We deduce properties of this measure on , and then of the product Lebesgue measure on ℝⁿ. In particular, we prove that they are translation invariant.

We show that, on ℝⁿ, a linear map acts on Lebesgue measure by rescaling it through the absolute value of its determinant, in Real.map_linearMap_volume_pi_eq_smul_volume_pi.

More properties of the Lebesgue measure are deduced from this in Mathlib/MeasureTheory/Measure/Lebesgue/EqHaar.lean, where they are proved more generally for any additive Haar measure on a finite-dimensional real vector space.

Definition of the Lebesgue measure and lengths of intervals #

The volume on the real line (as a particular case of the volume on a finite-dimensional inner product space) coincides with the Stieltjes measure coming from the identity function.

Volume of a box in ℝⁿ #

theorem Real.volume_Icc_pi {ι : Type u_1} [Fintype ι] {a b : ι} :
MeasureTheory.volume (Set.Icc a b) = i : ι, ENNReal.ofReal (b i - a i)
@[simp]
theorem Real.volume_Icc_pi_toReal {ι : Type u_1} [Fintype ι] {a b : ι} (h : a b) :
(MeasureTheory.volume (Set.Icc a b)).toReal = i : ι, (b i - a i)
theorem Real.volume_pi_Ioo {ι : Type u_1} [Fintype ι] {a b : ι} :
MeasureTheory.volume (Set.univ.pi fun (i : ι) => Set.Ioo (a i) (b i)) = i : ι, ENNReal.ofReal (b i - a i)
@[simp]
theorem Real.volume_pi_Ioo_toReal {ι : Type u_1} [Fintype ι] {a b : ι} (h : a b) :
(MeasureTheory.volume (Set.univ.pi fun (i : ι) => Set.Ioo (a i) (b i))).toReal = i : ι, (b i - a i)
theorem Real.volume_pi_Ioc {ι : Type u_1} [Fintype ι] {a b : ι} :
MeasureTheory.volume (Set.univ.pi fun (i : ι) => Set.Ioc (a i) (b i)) = i : ι, ENNReal.ofReal (b i - a i)
@[simp]
theorem Real.volume_pi_Ioc_toReal {ι : Type u_1} [Fintype ι] {a b : ι} (h : a b) :
(MeasureTheory.volume (Set.univ.pi fun (i : ι) => Set.Ioc (a i) (b i))).toReal = i : ι, (b i - a i)
theorem Real.volume_pi_Ico {ι : Type u_1} [Fintype ι] {a b : ι} :
MeasureTheory.volume (Set.univ.pi fun (i : ι) => Set.Ico (a i) (b i)) = i : ι, ENNReal.ofReal (b i - a i)
@[simp]
theorem Real.volume_pi_Ico_toReal {ι : Type u_1} [Fintype ι] {a b : ι} (h : a b) :
(MeasureTheory.volume (Set.univ.pi fun (i : ι) => Set.Ico (a i) (b i))).toReal = i : ι, (b i - a i)
@[simp]
theorem Real.volume_pi_ball {ι : Type u_1} [Fintype ι] (a : ι) {r : } (hr : 0 < r) :
@[simp]
theorem Real.volume_pi_closedBall {ι : Type u_1} [Fintype ι] (a : ι) {r : } (hr : 0 r) :
theorem Real.volume_pi_le_prod_diam {ι : Type u_1} [Fintype ι] (s : Set (ι)) :

Images of the Lebesgue measure under multiplication in ℝ #

Images of the Lebesgue measure under translation/linear maps in ℝⁿ #

A diagonal matrix rescales Lebesgue according to its determinant. This is a special case of Real.map_matrix_volume_pi_eq_smul_volume_pi, that one should use instead (and whose proof uses this particular case).

Any invertible matrix rescales Lebesgue measure through the absolute value of its determinant.

Any invertible linear map rescales Lebesgue measure through the absolute value of its determinant.

def regionBetween {α : Type u_1} (f g : α) (s : Set α) :
Set (α × )

The region between two real-valued functions on an arbitrary set.

Equations
Instances For
    theorem regionBetween_subset {α : Type u_1} (f g : α) (s : Set α) :
    theorem measurableSet_regionBetween {α : Type u_1} [MeasurableSpace α] {f g : α} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :

    The region between two measurable functions on a measurable set is measurable.

    theorem measurableSet_region_between_oc {α : Type u_1} [MeasurableSpace α] {f g : α} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    MeasurableSet {p : α × | p.1 s p.2 Set.Ioc (f p.1) (g p.1)}

    The region between two measurable functions on a measurable set is measurable; a version for the region together with the graph of the upper function.

    theorem measurableSet_region_between_co {α : Type u_1} [MeasurableSpace α] {f g : α} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    MeasurableSet {p : α × | p.1 s p.2 Set.Ico (f p.1) (g p.1)}

    The region between two measurable functions on a measurable set is measurable; a version for the region together with the graph of the lower function.

    theorem measurableSet_region_between_cc {α : Type u_1} [MeasurableSpace α] {f g : α} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    MeasurableSet {p : α × | p.1 s p.2 Set.Icc (f p.1) (g p.1)}

    The region between two measurable functions on a measurable set is measurable; a version for the region together with the graphs of both functions.

    theorem measurableSet_graph {α : Type u_1} [MeasurableSpace α] {f : α} (hf : Measurable f) :
    MeasurableSet {p : α × | p.2 = f p.1}

    The graph of a measurable function is a measurable set.

    theorem volume_regionBetween_eq_lintegral' {α : Type u_1} [MeasurableSpace α] {μ : MeasureTheory.Measure α} {f g : α} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    (μ.prod MeasureTheory.volume) (regionBetween f g s) = ∫⁻ (y : α) in s, ENNReal.ofReal ((g - f) y) μ
    theorem volume_regionBetween_eq_lintegral {α : Type u_1} [MeasurableSpace α] {μ : MeasureTheory.Measure α} {f g : α} {s : Set α} [MeasureTheory.SFinite μ] (hf : AEMeasurable f (μ.restrict s)) (hg : AEMeasurable g (μ.restrict s)) (hs : MeasurableSet s) :
    (μ.prod MeasureTheory.volume) (regionBetween f g s) = ∫⁻ (y : α) in s, ENNReal.ofReal ((g - f) y) μ

    The volume of the region between two almost everywhere measurable functions on a measurable set can be represented as a Lebesgue integral.

    theorem nullMeasurableSet_regionBetween {α : Type u_1} [MeasurableSpace α] (μ : MeasureTheory.Measure α) {f g : α} (f_mble : AEMeasurable f μ) (g_mble : AEMeasurable g μ) {s : Set α} (s_mble : MeasureTheory.NullMeasurableSet s μ) :

    The region between two a.e.-measurable functions on a null-measurable set is null-measurable.

    theorem nullMeasurableSet_region_between_oc {α : Type u_1} [MeasurableSpace α] (μ : MeasureTheory.Measure α) {f g : α} (f_mble : AEMeasurable f μ) (g_mble : AEMeasurable g μ) {s : Set α} (s_mble : MeasureTheory.NullMeasurableSet s μ) :

    The region between two a.e.-measurable functions on a null-measurable set is null-measurable; a version for the region together with the graph of the upper function.

    theorem nullMeasurableSet_region_between_co {α : Type u_1} [MeasurableSpace α] (μ : MeasureTheory.Measure α) {f g : α} (f_mble : AEMeasurable f μ) (g_mble : AEMeasurable g μ) {s : Set α} (s_mble : MeasureTheory.NullMeasurableSet s μ) :

    The region between two a.e.-measurable functions on a null-measurable set is null-measurable; a version for the region together with the graph of the lower function.

    theorem nullMeasurableSet_region_between_cc {α : Type u_1} [MeasurableSpace α] (μ : MeasureTheory.Measure α) {f g : α} (f_mble : AEMeasurable f μ) (g_mble : AEMeasurable g μ) {s : Set α} (s_mble : MeasureTheory.NullMeasurableSet s μ) :

    The region between two a.e.-measurable functions on a null-measurable set is null-measurable; a version for the region together with the graphs of both functions.

    theorem ae_restrict_of_ae_restrict_inter_Ioo {μ : MeasureTheory.Measure } [MeasureTheory.NoAtoms μ] {s : Set } {p : Prop} (h : ∀ (a b : ), a sb sa < b∀ᵐ (x : ) μ.restrict (s Set.Ioo a b), p x) :
    ∀ᵐ (x : ) μ.restrict s, p x

    Consider a real set s. If a property is true almost everywhere in s ∩ (a, b) for all a, b ∈ s, then it is true almost everywhere in s. Formulated with μ.restrict. See also ae_of_mem_of_ae_of_mem_inter_Ioo.

    theorem ae_of_mem_of_ae_of_mem_inter_Ioo {μ : MeasureTheory.Measure } [MeasureTheory.NoAtoms μ] {s : Set } {p : Prop} (h : ∀ (a b : ), a sb sa < b∀ᵐ (x : ) μ, x s Set.Ioo a bp x) :
    ∀ᵐ (x : ) μ, x sp x

    Consider a real set s. If a property is true almost everywhere in s ∩ (a, b) for all a, b ∈ s, then it is true almost everywhere in s. Formulated with bare membership. See also ae_restrict_of_ae_restrict_inter_Ioo.