mathlib3 documentation

measure_theory.measure.lebesgue.basic

Lebesgue measure on the real line and on ℝⁿ #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

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_linear_map_volume_pi_eq_smul_volume_pi.

More properties of the Lebesgue measure are deduced from this in lebesgue.eq_haar.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 : ι } :
@[simp]
theorem real.volume_Icc_pi_to_real {ι : Type u_1} [fintype ι] {a b : ι } (h : a b) :
theorem real.volume_pi_Ioo {ι : Type u_1} [fintype ι] {a b : ι } :
measure_theory.measure_space.volume (set.univ.pi (λ (i : ι), set.Ioo (a i) (b i))) = finset.univ.prod (λ (i : ι), ennreal.of_real (b i - a i))
@[simp]
theorem real.volume_pi_Ioo_to_real {ι : Type u_1} [fintype ι] {a b : ι } (h : a b) :
(measure_theory.measure_space.volume (set.univ.pi (λ (i : ι), set.Ioo (a i) (b i)))).to_real = finset.univ.prod (λ (i : ι), b i - a i)
theorem real.volume_pi_Ioc {ι : Type u_1} [fintype ι] {a b : ι } :
measure_theory.measure_space.volume (set.univ.pi (λ (i : ι), set.Ioc (a i) (b i))) = finset.univ.prod (λ (i : ι), ennreal.of_real (b i - a i))
@[simp]
theorem real.volume_pi_Ioc_to_real {ι : Type u_1} [fintype ι] {a b : ι } (h : a b) :
(measure_theory.measure_space.volume (set.univ.pi (λ (i : ι), set.Ioc (a i) (b i)))).to_real = finset.univ.prod (λ (i : ι), b i - a i)
theorem real.volume_pi_Ico {ι : Type u_1} [fintype ι] {a b : ι } :
measure_theory.measure_space.volume (set.univ.pi (λ (i : ι), set.Ico (a i) (b i))) = finset.univ.prod (λ (i : ι), ennreal.of_real (b i - a i))
@[simp]
theorem real.volume_pi_Ico_to_real {ι : Type u_1} [fintype ι] {a b : ι } (h : a b) :
(measure_theory.measure_space.volume (set.univ.pi (λ (i : ι), set.Ico (a i) (b i)))).to_real = finset.univ.prod (λ (i : ι), b i - a i)
@[simp]
theorem real.volume_pi_ball {ι : Type u_1} [fintype ι] (a : ι ) {r : } (hr : 0 < r) :
@[simp]

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 region_between {α : Type u_1} (f g : α ) (s : set α) :
set × )

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

Equations
theorem region_between_subset {α : Type u_1} (f g : α ) (s : set α) :
theorem measurable_set_region_between {α : Type u_1} [measurable_space α] {f g : α } {s : set α} (hf : measurable f) (hg : measurable g) (hs : measurable_set s) :

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

theorem measurable_set_region_between_oc {α : Type u_1} [measurable_space α] {f g : α } {s : set α} (hf : measurable f) (hg : measurable g) (hs : measurable_set s) :
measurable_set {p : α × | p.fst s p.snd set.Ioc (f p.fst) (g p.fst)}

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 measurable_set_region_between_co {α : Type u_1} [measurable_space α] {f g : α } {s : set α} (hf : measurable f) (hg : measurable g) (hs : measurable_set s) :
measurable_set {p : α × | p.fst s p.snd set.Ico (f p.fst) (g p.fst)}

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 measurable_set_region_between_cc {α : Type u_1} [measurable_space α] {f g : α } {s : set α} (hf : measurable f) (hg : measurable g) (hs : measurable_set s) :
measurable_set {p : α × | p.fst s p.snd set.Icc (f p.fst) (g p.fst)}

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 measurable_set_graph {α : Type u_1} [measurable_space α] {f : α } (hf : measurable f) :
measurable_set {p : α × | p.snd = f p.fst}

The graph of a measurable function is a measurable set.

theorem volume_region_between_eq_lintegral' {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f g : α } {s : set α} (hf : measurable f) (hg : measurable g) (hs : measurable_set s) :

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

theorem ae_restrict_of_ae_restrict_inter_Ioo {μ : measure_theory.measure } [measure_theory.has_no_atoms μ] {s : set } {p : Prop} (h : (a b : ), a s b s a < 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 {μ : measure_theory.measure } [measure_theory.has_no_atoms μ] {s : set } {p : Prop} (h : (a b : ), a s b s a < b (∀ᵐ (x : ) μ, x s set.Ioo a b p x)) :
∀ᵐ (x : ) μ, x 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 bare membership. See also ae_restrict_of_ae_restrict_inter_Ioo.