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 : ιReal} :
theorem Real.volume_Icc_pi_toReal {ι : Type u_1} [Fintype ι] {a b : ιReal} (h : LE.le a b) :
theorem Real.volume_pi_Ioo {ι : Type u_1} [Fintype ι] {a b : ιReal} :
Eq (DFunLike.coe MeasureTheory.MeasureSpace.volume (Set.univ.pi fun (i : ι) => Set.Ioo (a i) (b i))) (Finset.univ.prod fun (i : ι) => ENNReal.ofReal (HSub.hSub (b i) (a i)))
theorem Real.volume_pi_Ioo_toReal {ι : Type u_1} [Fintype ι] {a b : ιReal} (h : LE.le a b) :
Eq (DFunLike.coe MeasureTheory.MeasureSpace.volume (Set.univ.pi fun (i : ι) => Set.Ioo (a i) (b i))).toReal (Finset.univ.prod fun (i : ι) => HSub.hSub (b i) (a i))
theorem Real.volume_pi_Ioc {ι : Type u_1} [Fintype ι] {a b : ιReal} :
Eq (DFunLike.coe MeasureTheory.MeasureSpace.volume (Set.univ.pi fun (i : ι) => Set.Ioc (a i) (b i))) (Finset.univ.prod fun (i : ι) => ENNReal.ofReal (HSub.hSub (b i) (a i)))
theorem Real.volume_pi_Ioc_toReal {ι : Type u_1} [Fintype ι] {a b : ιReal} (h : LE.le a b) :
Eq (DFunLike.coe MeasureTheory.MeasureSpace.volume (Set.univ.pi fun (i : ι) => Set.Ioc (a i) (b i))).toReal (Finset.univ.prod fun (i : ι) => HSub.hSub (b i) (a i))
theorem Real.volume_pi_Ico {ι : Type u_1} [Fintype ι] {a b : ιReal} :
Eq (DFunLike.coe MeasureTheory.MeasureSpace.volume (Set.univ.pi fun (i : ι) => Set.Ico (a i) (b i))) (Finset.univ.prod fun (i : ι) => ENNReal.ofReal (HSub.hSub (b i) (a i)))
theorem Real.volume_pi_Ico_toReal {ι : Type u_1} [Fintype ι] {a b : ιReal} (h : LE.le a b) :
Eq (DFunLike.coe MeasureTheory.MeasureSpace.volume (Set.univ.pi fun (i : ι) => Set.Ico (a i) (b i))).toReal (Finset.univ.prod fun (i : ι) => HSub.hSub (b i) (a i))

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 : αReal) (s : Set α) :

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

Equations
Instances For
    theorem regionBetween_subset {α : Type u_1} (f g : αReal) (s : Set α) :
    theorem measurableSet_regionBetween {α : Type u_1} [MeasurableSpace α] {f g : αReal} {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 : αReal} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    MeasurableSet (setOf fun (p : Prod α Real) => And (Membership.mem s p.fst) (Membership.mem (Set.Ioc (f p.fst) (g p.fst)) p.snd))

    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 : αReal} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    MeasurableSet (setOf fun (p : Prod α Real) => And (Membership.mem s p.fst) (Membership.mem (Set.Ico (f p.fst) (g p.fst)) p.snd))

    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 : αReal} {s : Set α} (hf : Measurable f) (hg : Measurable g) (hs : MeasurableSet s) :
    MeasurableSet (setOf fun (p : Prod α Real) => And (Membership.mem s p.fst) (Membership.mem (Set.Icc (f p.fst) (g p.fst)) p.snd))

    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 : αReal} (hf : Measurable f) :
    MeasurableSet (setOf fun (p : Prod α Real) => Eq p.snd (f p.fst))

    The graph of a measurable function is a measurable set.

    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 : αReal} (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.

    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.

    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.

    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 Real} [MeasureTheory.NoAtoms μ] {s : Set Real} {p : RealProp} (h : ∀ (a b : Real), Membership.mem s aMembership.mem s bLT.lt a bFilter.Eventually (fun (x : Real) => p x) (MeasureTheory.ae (μ.restrict (Inter.inter s (Set.Ioo a b))))) :
    Filter.Eventually (fun (x : Real) => p x) (MeasureTheory.ae (μ.restrict s))

    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 Real} [MeasureTheory.NoAtoms μ] {s : Set Real} {p : RealProp} (h : ∀ (a b : Real), Membership.mem s aMembership.mem s bLT.lt a bFilter.Eventually (fun (x : Real) => Membership.mem (Inter.inter s (Set.Ioo a b)) xp x) (MeasureTheory.ae μ)) :
    Filter.Eventually (fun (x : Real) => Membership.mem s xp x) (MeasureTheory.ae μ)

    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.