mathlib documentation

measure_theory.​bochner_integration

measure_theory.​bochner_integration

Bochner integral

The Bochner integral extends the definition of the Lebesgue integral to functions that map from a measure space into a Banach space (complete normed vector space). It is constructed here by extending the integral on simple functions.

Main definitions

The Bochner integral is defined following these steps:

  1. Define the integral on simple functions of the type simple_func α E (notation : α →ₛ E) where E is a real normed space.

    (See simple_func.bintegral and section bintegral for details. Also see simple_func.integral for the integral on simple functions of the type simple_func α ennreal.)

  2. Use α →ₛ E to cut out the simple functions from L1 functions, and define integral on these. The type of simple functions in L1 space is written as α →₁ₛ[μ] E.

  3. Show that the embedding of α →₁ₛ[μ] E into L1 is a dense and uniform one.

  4. Show that the integral defined on α →₁ₛ[μ] E is a continuous linear map.

  5. Define the Bochner integral on L1 functions by extending the integral on integrable simple functions α →₁ₛ[μ] E using continuous_linear_map.extend. Define the Bochner integral on functions as the Bochner integral of its equivalence class in L1 space.

Main statements

  1. Basic properties of the Bochner integral on functions of type α → E, where α is a measure space and E is a real normed space.

    • integral_zero : ∫ 0 = 0
    • integral_add : ∫ f + g = ∫ f + ∫ g
    • integral_neg : ∫ -f = - ∫ f
    • integral_sub : ∫ f - g = ∫ f - ∫ g
    • integral_smul : ∫ r • f = r • ∫ f
    • integral_congr_ae : ∀ᵐ a, f a = g a → ∫ f = ∫ g
    • norm_integral_le_integral_norm : ∥∫ f∥ ≤ ∫ ∥f∥
  2. Basic properties of the Bochner integral on functions of type α → ℝ, where α is a measure space.

    • integral_nonneg_of_ae : ∀ᵐ a, 0 ≤ f a → 0 ≤ ∫ f
    • integral_nonpos_of_nonpos_ae : ∀ᵐ a, f a ≤ 0 → ∫ f ≤ 0
    • integral_le_integral_of_le_ae : ∀ᵐ a, f a ≤ g a → ∫ f ≤ ∫ g
  3. Propositions connecting the Bochner integral with the integral on ennreal-valued functions, which is called lintegral and has the notation ∫⁻.

    • integral_eq_lintegral_max_sub_lintegral_min : ∫ f = ∫⁻ f⁺ - ∫⁻ f⁻, where f⁺ is the positive part of f and f⁻ is the negative part of f.
    • integral_eq_lintegral_of_nonneg_ae : ∀ᵐ a, 0 ≤ f a → ∫ f = ∫⁻ f
  4. tendsto_integral_of_dominated_convergence : the Lebesgue dominated convergence theorem

Notes

Some tips on how to prove a proposition if the API for the Bochner integral is not enough so that you need to unfold the definition of the Bochner integral and go back to simple functions.

See integral_eq_lintegral_max_sub_lintegral_min for a complicated example, which proves that ∫ f = ∫⁻ f⁺ - ∫⁻ f⁻, with the first integral sign being the Bochner integral of a real-valued function f : α → ℝ, and second and third integral sign being the integral on ennreal-valued functions (called lintegral). The proof of integral_eq_lintegral_max_sub_lintegral_min is scattered in sections with the name pos_part.

Here are the usual steps of proving that a property p, say ∫ f = ∫⁻ f⁺ - ∫⁻ f⁻, holds for all functions :

  1. First go to the space.

    For example, if you see ennreal.to_real (∫⁻ a, ennreal.of_real $ ∥f a∥), that is the norm of f in space. Rewrite using l1.norm_of_fun_eq_lintegral_norm.

  2. Show that the set {f ∈ L¹ | ∫ f = ∫⁻ f⁺ - ∫⁻ f⁻} is closed in using is_closed_eq.

  3. Show that the property holds for all simple functions s in space.

    Typically, you need to convert various notions to their simple_func counterpart, using lemmas like l1.integral_coe_eq_integral.

  4. Since simple functions are dense in ,

univ = closure {s simple}
     = closure {s simple |  s = ∫⁻ s - ∫⁻ s} : the property holds for all simple functions
      closure {f |  f = ∫⁻ f - ∫⁻ f}
     = {f |  f = ∫⁻ f - ∫⁻ f} : closure of a closed set is itself

Use is_closed_property or dense_range.induction_on for this argument.

Notations

Note : is typed using \_s. Sometimes it shows as a box if font is missing.

Tags

Bochner integral, simple function, function space, Lebesgue dominated convergence theorem

Positive part of a simple function.

Equations

Negative part of a simple function.

Equations

The Bochner integral of simple functions

Define the Bochner integral of simple functions of the type α →ₛ β where β is a normed group, and prove basic property of this integral.

For simple functions with a normed_group as codomain, being integrable is the same as having finite volume support.

Bochner integral of simple functions whose codomain is a real normed_space.

Equations
theorem measure_theory.​simple_func.​map_integral {α : Type u_1} {E : Type u_2} {F : Type u_3} [measurable_space α] [normed_group E] [normed_group F] {μ : measure_theory.measure α} [normed_space F] (f : measure_theory.simple_func α E) (g : E → F) :

Calculate the integral of g ∘ f : α →ₛ F, where f is an integrable function from α to E and g is a function from E to F. We require g 0 = 0 so that g ∘ f is integrable.

simple_func.integral and simple_func.lintegral agree when the integrand has type α →ₛ ennreal. But since ennreal is not a normed_space, we need some form of coercion. See integral_eq_lintegral for a simpler version.

simple_func.bintegral and simple_func.integral agree when the integrand has type α →ₛ ennreal. But since ennreal is not a normed_space, we need some form of coercion.

l1.simple_func is a subspace of L1 consisting of equivalence classes of an integrable simple function.

Equations

Simple functions in L1 space form a normed_space.

L1 simple functions forms a emetric_space, with the emetric being inherited from L1 space, i.e., edist f g = ∫⁻ a, edist (f a) (g a). Not declared as an instance as α →₁ₛ[μ] β will only be useful in the construction of the bochner integral.

Equations

L1 simple functions forms a metric_space, with the metric being inherited from L1 space, i.e., dist f g = ennreal.to_real (∫⁻ a, edist (f a) (g a)). Not declared as an instance as α →₁ₛ[μ] β will only be useful in the construction of the bochner integral.

Equations

The norm on α →₁ₛ[μ] E is inherited from L1 space. That is, ∥f∥ = ∫⁻ a, edist (f a) 0. Not declared as an instance as α →₁ₛ[μ] E will only be useful in the construction of the bochner integral.

Equations

Not declared as an instance as α →₁ₛ[μ] E will only be useful in the construction of the bochner integral.

Equations

Not declared as an instance as α →₁ₛ[μ] E will only be useful in the construction of the bochner integral.

Equations
@[simp]
theorem measure_theory.​l1.​simple_func.​coe_smul {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {𝕜 : Type u_4} [normed_field 𝕜] [normed_space 𝕜 E] (c : 𝕜) (f : α →₁ₛ[μ] E) :
(c f) = c f

Not declared as an instance as α →₁ₛ[μ] E will only be useful in the construction of the bochner integral.

Equations

Not declared as an instance as α →₁ₛ[μ] E will only be useful in the construction of the bochner integral.

Equations

Construct the equivalence class [f] of an integrable simple function f.

Equations

The uniform and dense embedding of L1 simple functions into L1 functions.

Equations

Positive part of a simple function in L1 space.

Equations

Negative part of a simple function in L1 space.

Equations

Define the Bochner integral on α →₁ₛ[μ] E and prove basic properties of this integral.

The Bochner integral over simple functions in l1 space.

Equations

The Bochner integral over simple functions in l1 space as a continuous linear map.

Equations
theorem measure_theory.​integral_add {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {f g : α → E} {μ : measure_theory.measure α} :
measurable fmeasure_theory.integrable f μmeasurable gmeasure_theory.integrable g μ (a : α), f a + g a μ = (a : α), f a μ + (a : α), g a μ

theorem measure_theory.​integral_neg {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} (f : α → E) :
(a : α), -f a μ = - (a : α), f a μ

theorem measure_theory.​integral_sub {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {f g : α → E} {μ : measure_theory.measure α} :
measurable fmeasure_theory.integrable f μmeasurable gmeasure_theory.integrable g μ (a : α), f a - g a μ = (a : α), f a μ - (a : α), g a μ

theorem measure_theory.​integral_smul {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} (r : ) (f : α → E) :
(a : α), r f a μ = r (a : α), f a μ

theorem measure_theory.​integral_mul_left {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} (r : ) (f : α → ) :
(a : α), r * f a μ = r * (a : α), f a μ

theorem measure_theory.​integral_mul_right {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} (r : ) (f : α → ) :
(a : α), f a * r μ = (a : α), f a μ * r

theorem measure_theory.​integral_div {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} (r : ) (f : α → ) :
(a : α), f a / r μ = (a : α), f a μ / r

theorem measure_theory.​integral_congr_ae {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {f g : α → E} {μ : measure_theory.measure α} :
measurable fmeasurable gf =ᵐ[μ] g (a : α), f a μ = (a : α), g a μ

theorem measure_theory.​tendsto_integral_of_l1 {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {ι : Type u_3} (f : α → E) (hfm : measurable f) (hfi : measure_theory.integrable f μ) {F : ι → α → E} {l : filter ι} :
(∀ᶠ (i : ι) in l, measurable (F i))(∀ᶠ (i : ι) in l, measure_theory.integrable (F i) μ)filter.tendsto (λ (i : ι), ∫⁻ (x : α), has_edist.edist (F i x) (f x) μ) l (nhds 0)filter.tendsto (λ (i : ι), (x : α), F i x μ) l (nhds ( (x : α), f x μ))

If F i → f in L1, then ∫ x, F i x ∂μ → ∫ x, f x∂μ.

theorem measure_theory.​tendsto_integral_of_dominated_convergence {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {F : α → E} {f : α → E} (bound : α → ) :
(∀ (n : ), measurable (F n))measurable fmeasure_theory.integrable bound μ(∀ (n : ), ∀ᵐ (a : α) ∂μ, F n a bound a)(∀ᵐ (a : α) ∂μ, filter.tendsto (λ (n : ), F n a) filter.at_top (nhds (f a)))filter.tendsto (λ (n : ), (a : α), F n a μ) filter.at_top (nhds ( (a : α), f a μ))

Lebesgue dominated convergence theorem provides sufficient conditions under which almost everywhere convergence of a sequence of functions implies the convergence of their integrals.

theorem measure_theory.​tendsto_integral_filter_of_dominated_convergence {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {ι : Type u_3} {l : filter ι} {F : ι → α → E} {f : α → E} (bound : α → ) :
l.is_countably_generated(∀ᶠ (n : ι) in l, measurable (F n))measurable f(∀ᶠ (n : ι) in l, ∀ᵐ (a : α) ∂μ, F n a bound a)measure_theory.integrable bound μ(∀ᵐ (a : α) ∂μ, filter.tendsto (λ (n : ι), F n a) l (nhds (f a)))filter.tendsto (λ (n : ι), (a : α), F n a μ) l (nhds ( (a : α), f a μ))

Lebesgue dominated convergence theorem for filters with a countable basis

theorem measure_theory.​integral_eq_lintegral_max_sub_lintegral_min {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f : α → } :
measurable fmeasure_theory.integrable f μ (a : α), f a μ = (∫⁻ (a : α), ennreal.of_real (max (f a) 0) μ).to_real - (∫⁻ (a : α), ennreal.of_real (-min (f a) 0) μ).to_real

The Bochner integral of a real-valued function f : α → ℝ is the difference between the integral of the positive part of f and the integral of the negative part of f.

theorem measure_theory.​integral_eq_lintegral_of_nonneg_ae {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f : α → } :
0 ≤ᵐ[μ] fmeasurable f (a : α), f a μ = (∫⁻ (a : α), ennreal.of_real (f a) μ).to_real

theorem measure_theory.​integral_nonneg_of_ae {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f : α → } :
0 ≤ᵐ[μ] f0 (a : α), f a μ

theorem measure_theory.​integral_nonpos_of_nonpos_ae {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f : α → } :
f ≤ᵐ[μ] 0 (a : α), f a μ 0

theorem measure_theory.​integral_mono {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f g : α → } :
measurable fmeasure_theory.integrable f μmeasurable gmeasure_theory.integrable g μf ≤ᵐ[μ] g (a : α), f a μ (a : α), g a μ

theorem measure_theory.​integral_mono_of_nonneg {α : Type u_1} [measurable_space α] {μ : measure_theory.measure α} {f g : α → } :
0 ≤ᵐ[μ] fmeasurable gmeasure_theory.integrable g μf ≤ᵐ[μ] g (a : α), f a μ (a : α), g a μ

theorem measure_theory.​norm_integral_le_of_norm_le {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {f : α → E} {g : α → } :
measurable gmeasure_theory.integrable g μ(∀ᵐ (x : α) ∂μ, f x g x) (x : α), f x μ (x : α), g x μ

theorem measure_theory.​integral_finset_sum {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {ι : Type u_3} (s : finset ι) {f : ι → α → E} :
(∀ (i : ι), measurable (f i))(∀ (i : ι), measure_theory.integrable (f i) μ) (a : α), s.sum (λ (i : ι), f i a) μ = s.sum (λ (i : ι), (a : α), f i a μ)

theorem measure_theory.​integral_add_measure {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ ν : measure_theory.measure α} {f : α → E} :
measure_theory.integrable f μmeasure_theory.integrable f ν (x : α), f x + ν) = (x : α), f x μ + (x : α), f x ν

@[simp]

@[simp]
theorem measure_theory.​integral_smul_measure {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} (f : α → E) (c : ennreal) :
(x : α), f x c μ = c.to_real (x : α), f x μ

theorem measure_theory.​integral_map_measure {α : Type u_1} {E : Type u_2} [measurable_space α] [normed_group E] [topological_space.second_countable_topology E] [normed_space E] [complete_space E] [measurable_space E] [borel_space E] {μ : measure_theory.measure α} {β : Type u_3} [measurable_space β] {φ : α → β} (hφ : measurable φ) {f : β → E} :
measurable f (y : β), f y (measure_theory.measure.map φ) μ = (x : α), f (φ x) μ