Documentation

Mathlib.MeasureTheory.Integral.Layercake

The layer cake formula / Cavalieri's principle / tail probability formula #

In this file we prove the following layer cake formula.

Consider a non-negative measurable function f on a measure space. Apply pointwise to it an increasing absolutely continuous function G : ℝ≥0 → ℝ≥0 vanishing at the origin, with derivative G' = g on the positive real line (in other words, G a primitive of a non-negative locally integrable function g on the positive real line). Then the integral of the result, ∫ G ∘ f, can be written as the integral over the positive real line of the "tail measures" of f (i.e., a function giving the measures of the sets on which f exceeds different positive real values) weighted by g. In probability theory contexts, the "tail measures" could be referred to as "tail probabilities" of the random variable f, or as values of the "complementary cumulative distribution function" of the random variable f. The terminology "tail probability formula" is therefore occasionally used for the layer cake formula (or a standard application of it).

The essence of the (mathematical) proof is Fubini's theorem.

We also give the two most common applications of the layer cake formula

Variants of the formulas with measures of sets of the form {ω | f(ω) > t} instead of {ω | f(ω) ≥ t} are also included.

Main results #

Tags #

layer cake representation, Cavalieri's principle, tail probability formula

theorem MeasureTheory.countable_meas_le_ne_meas_lt {α : Type u_1} {R : Type u_2} [MeasurableSpace α] (μ : MeasureTheory.Measure α) [LinearOrder R] (g : αR) :
Set.Countable {t : R | μ {a : α | t g a} μ {a : α | t < g a}}
theorem MeasureTheory.meas_le_ae_eq_meas_lt {α : Type u_1} [MeasurableSpace α] (μ : MeasureTheory.Measure α) {R : Type u_3} [LinearOrder R] [MeasurableSpace R] (ν : MeasureTheory.Measure R) [MeasureTheory.NoAtoms ν] (g : αR) :
(fun (t : R) => μ {a : α | t g a}) =ᶠ[MeasureTheory.Measure.ae ν] fun (t : R) => μ {a : α | t < g a}

Layercake formula #

theorem MeasureTheory.lintegral_comp_eq_lintegral_meas_le_mul_of_measurable_of_sigmaFinite {α : Type u_1} [MeasurableSpace α] {f : α} {g : } (μ : MeasureTheory.Measure α) [MeasureTheory.SigmaFinite μ] (f_nn : 0 f) (f_mble : Measurable f) (g_intble : t > 0, IntervalIntegrable g MeasureTheory.volume 0 t) (g_mble : Measurable g) (g_nn : t > 0, 0 g t) :
∫⁻ (ω : α), ENNReal.ofReal (∫ (t : ) in 0 ..f ω, g t)μ = ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t f a} * ENNReal.ofReal (g t)

An auxiliary version of the layer cake formula (Cavalieri's principle, tail probability formula), with a measurability assumption that would also essentially follow from the integrability assumptions, and a sigma-finiteness assumption.

See MeasureTheory.lintegral_comp_eq_lintegral_meas_le_mul and MeasureTheory.lintegral_comp_eq_lintegral_meas_lt_mul for the main formulations of the layer cake formula.

theorem MeasureTheory.lintegral_comp_eq_lintegral_meas_le_mul_of_measurable {α : Type u_1} [MeasurableSpace α] {f : α} {g : } (μ : MeasureTheory.Measure α) (f_nn : 0 f) (f_mble : Measurable f) (g_intble : t > 0, IntervalIntegrable g MeasureTheory.volume 0 t) (g_mble : Measurable g) (g_nn : t > 0, 0 g t) :
∫⁻ (ω : α), ENNReal.ofReal (∫ (t : ) in 0 ..f ω, g t)μ = ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t f a} * ENNReal.ofReal (g t)

An auxiliary version of the layer cake formula (Cavalieri's principle, tail probability formula), with a measurability assumption that would also essentially follow from the integrability assumptions. Compared to lintegral_comp_eq_lintegral_meas_le_mul_of_measurable_of_sigmaFinite, we remove the sigma-finite assumption.

See MeasureTheory.lintegral_comp_eq_lintegral_meas_le_mul and MeasureTheory.lintegral_comp_eq_lintegral_meas_lt_mul for the main formulations of the layer cake formula.

theorem MeasureTheory.lintegral_comp_eq_lintegral_meas_le_mul {α : Type u_1} [MeasurableSpace α] {f : α} {g : } (μ : MeasureTheory.Measure α) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_mble : AEMeasurable f μ) (g_intble : t > 0, IntervalIntegrable g MeasureTheory.volume 0 t) (g_nn : ∀ᵐ (t : ) ∂MeasureTheory.volume.restrict (Set.Ioi 0), 0 g t) :
∫⁻ (ω : α), ENNReal.ofReal (∫ (t : ) in 0 ..f ω, g t)μ = ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t f a} * ENNReal.ofReal (g t)

The layer cake formula / Cavalieri's principle / tail probability formula:

Let f be a non-negative measurable function on a measure space. Let G be an increasing absolutely continuous function on the positive real line, vanishing at the origin, with derivative G' = g. Then the integral of the composition G ∘ f can be written as the integral over the positive real line of the "tail measures" μ {ω | f(ω) ≥ t} of f weighted by g.

Roughly speaking, the statement is: ∫⁻ (G ∘ f) ∂μ = ∫⁻ t in 0..∞, g(t) * μ {ω | f(ω) ≥ t}.

See MeasureTheory.lintegral_comp_eq_lintegral_meas_lt_mul for a version with sets of the form {ω | f(ω) > t} instead.

theorem MeasureTheory.lintegral_eq_lintegral_meas_le {α : Type u_1} [MeasurableSpace α] {f : α} (μ : MeasureTheory.Measure α) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_mble : AEMeasurable f μ) :
∫⁻ (ω : α), ENNReal.ofReal (f ω)μ = ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t f a}

The standard case of the layer cake formula / Cavalieri's principle / tail probability formula:

For a nonnegative function f on a measure space, the Lebesgue integral of f can be written (roughly speaking) as: ∫⁻ f ∂μ = ∫⁻ t in 0..∞, μ {ω | f(ω) ≥ t}.

See MeasureTheory.lintegral_eq_lintegral_meas_lt for a version with sets of the form {ω | f(ω) > t} instead.

theorem MeasureTheory.lintegral_rpow_eq_lintegral_meas_le_mul {α : Type u_1} [MeasurableSpace α] {f : α} (μ : MeasureTheory.Measure α) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_mble : AEMeasurable f μ) {p : } (p_pos : 0 < p) :
∫⁻ (ω : α), ENNReal.ofReal (f ω ^ p)μ = ENNReal.ofReal p * ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t f a} * ENNReal.ofReal (t ^ (p - 1))

An application of the layer cake formula / Cavalieri's principle / tail probability formula:

For a nonnegative function f on a measure space, the Lebesgue integral of f can be written (roughly speaking) as: ∫⁻ f^p ∂μ = p * ∫⁻ t in 0..∞, t^(p-1) * μ {ω | f(ω) ≥ t}.

See MeasureTheory.lintegral_rpow_eq_lintegral_meas_lt_mul for a version with sets of the form {ω | f(ω) > t} instead.

theorem MeasureTheory.lintegral_comp_eq_lintegral_meas_lt_mul {α : Type u_1} [MeasurableSpace α] {f : α} {g : } (μ : MeasureTheory.Measure α) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_mble : AEMeasurable f μ) (g_intble : t > 0, IntervalIntegrable g MeasureTheory.volume 0 t) (g_nn : ∀ᵐ (t : ) ∂MeasureTheory.volume.restrict (Set.Ioi 0), 0 g t) :
∫⁻ (ω : α), ENNReal.ofReal (∫ (t : ) in 0 ..f ω, g t)μ = ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t < f a} * ENNReal.ofReal (g t)

The layer cake formula / Cavalieri's principle / tail probability formula:

Let f be a non-negative measurable function on a measure space. Let G be an increasing absolutely continuous function on the positive real line, vanishing at the origin, with derivative G' = g. Then the integral of the composition G ∘ f can be written as the integral over the positive real line of the "tail measures" μ {ω | f(ω) > t} of f weighted by g.

Roughly speaking, the statement is: ∫⁻ (G ∘ f) ∂μ = ∫⁻ t in 0..∞, g(t) * μ {ω | f(ω) > t}.

See lintegral_comp_eq_lintegral_meas_le_mul for a version with sets of the form {ω | f(ω) ≥ t} instead.

theorem MeasureTheory.lintegral_eq_lintegral_meas_lt {α : Type u_1} [MeasurableSpace α] {f : α} (μ : MeasureTheory.Measure α) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_mble : AEMeasurable f μ) :
∫⁻ (ω : α), ENNReal.ofReal (f ω)μ = ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t < f a}

The standard case of the layer cake formula / Cavalieri's principle / tail probability formula:

For a nonnegative function f on a measure space, the Lebesgue integral of f can be written (roughly speaking) as: ∫⁻ f ∂μ = ∫⁻ t in 0..∞, μ {ω | f(ω) > t}.

See lintegral_eq_lintegral_meas_le for a version with sets of the form {ω | f(ω) ≥ t} instead.

theorem MeasureTheory.lintegral_rpow_eq_lintegral_meas_lt_mul {α : Type u_1} [MeasurableSpace α] {f : α} (μ : MeasureTheory.Measure α) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_mble : AEMeasurable f μ) {p : } (p_pos : 0 < p) :
∫⁻ (ω : α), ENNReal.ofReal (f ω ^ p)μ = ENNReal.ofReal p * ∫⁻ (t : ) in Set.Ioi 0, μ {a : α | t < f a} * ENNReal.ofReal (t ^ (p - 1))

An application of the layer cake formula / Cavalieri's principle / tail probability formula:

For a nonnegative function f on a measure space, the Lebesgue integral of f can be written (roughly speaking) as: ∫⁻ f^p ∂μ = p * ∫⁻ t in 0..∞, t^(p-1) * μ {ω | f(ω) > t}.

See lintegral_rpow_eq_lintegral_meas_le_mul for a version with sets of the form {ω | f(ω) ≥ t} instead.

theorem MeasureTheory.Integrable.integral_eq_integral_meas_lt {α : Type u_1} [MeasurableSpace α] {μ : MeasureTheory.Measure α} {f : α} (f_intble : MeasureTheory.Integrable f μ) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) :
∫ (ω : α), f ωμ = ∫ (t : ) in Set.Ioi 0, (μ {a : α | t < f a}).toReal

The standard case of the layer cake formula / Cavalieri's principle / tail probability formula:

For an integrable a.e.-nonnegative real-valued function f, the Bochner integral of f can be written (roughly speaking) as: ∫ f ∂μ = ∫ t in 0..∞, μ {ω | f(ω) > t}.

See MeasureTheory.lintegral_eq_lintegral_meas_lt for a version with Lebesgue integral ∫⁻ instead.

theorem MeasureTheory.Integrable.integral_eq_integral_meas_le {α : Type u_1} [MeasurableSpace α] {μ : MeasureTheory.Measure α} {f : α} (f_intble : MeasureTheory.Integrable f μ) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) :
∫ (ω : α), f ωμ = ∫ (t : ) in Set.Ioi 0, (μ {a : α | t f a}).toReal
theorem MeasureTheory.Integrable.integral_eq_integral_Ioc_meas_le {α : Type u_1} [MeasurableSpace α] {μ : MeasureTheory.Measure α} {f : α} {M : } (f_intble : MeasureTheory.Integrable f μ) (f_nn : 0 ≤ᶠ[MeasureTheory.Measure.ae μ] f) (f_bdd : f ≤ᶠ[MeasureTheory.Measure.ae μ] fun (x : α) => M) :
∫ (ω : α), f ωμ = ∫ (t : ) in Set.Ioc 0 M, (μ {a : α | t f a}).toReal