mathlib3 documentation

measure_theory.integral.bochner

Bochner integral #

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

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 through the extension process described in the file set_to_L1, which follows these steps:

  1. Define the integral of the indicator of a set. This is weighted_smul μ s x = (μ s).to_real * x. weighted_smul μ is shown to be linear in the value x and dominated_fin_meas_additive (defined in the file set_to_L1) with respect to the set s.

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

  3. Transfer this definition to define the integral on L1.simple_func α E (notation : α →₁ₛ[μ] E), see L1.simple_func.integral. Show that this integral is a continuous linear map from α →₁ₛ[μ] E to E.

  4. Define the Bochner integral on L1 functions by extending the integral on integrable simple functions α →₁ₛ[μ] E using continuous_linear_map.extend and the fact that the embedding of α →₁ₛ[μ] E into α →₁[μ] E is dense.

  5. Define the Bochner integral on functions as the Bochner integral of its equivalence class in L1 space, if it is in L1, and 0 otherwise.

The result of that construction is ∫ a, f a ∂μ, which is definitionally equal to set_to_fun (dominated_fin_meas_additive_weighted_smul μ) f. Some basic properties of the integral (like linearity) are particular cases of the properties of set_to_fun (which are described in the file set_to_L1).

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.
  1. Basic properties of the Bochner integral on functions of type α → ℝ, where α is a measure space.
  1. Propositions connecting the Bochner integral with the integral on ℝ≥0∞-valued functions, which is called lintegral and has the notation ∫⁻.
  1. tendsto_integral_of_dominated_convergence : the Lebesgue dominated convergence theorem

  2. (In the file set_integral) integration commutes with continuous linear maps.

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.

One method is to use the theorem integrable.induction in the file simple_func_dense_lp (or one of the related results, like Lp.induction for functions in Lp), which allows you to prove something for an arbitrary integrable function.

Another method is using the following steps. 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 ℝ≥0∞-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 #

We also define notations for integral on a set, which are described in the file measure_theory/set_integral.

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

Tags #

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

noncomputable def measure_theory.weighted_smul {α : Type u_1} {F : Type u_3} [normed_add_comm_group F] [normed_space F] {m : measurable_space α} (μ : measure_theory.measure α) (s : set α) :

Given a set s, return the continuous linear map λ x, (μ s).to_real • x. The extension of that set function through set_to_L1 gives the Bochner integral of L1 functions.

Equations
theorem measure_theory.weighted_smul_null {α : Type u_1} {F : Type u_3} [normed_add_comm_group F] [normed_space F] {m : measurable_space α} {μ : measure_theory.measure α} {s : set α} (h_zero : μ s = 0) :
theorem measure_theory.weighted_smul_union' {α : Type u_1} {F : Type u_3} [normed_add_comm_group F] [normed_space F] {m : measurable_space α} {μ : measure_theory.measure α} (s t : set α) (ht : measurable_set t) (hs_finite : μ s ) (ht_finite : μ t ) (h_inter : s t = ) :
@[nolint]
theorem measure_theory.weighted_smul_union {α : Type u_1} {F : Type u_3} [normed_add_comm_group F] [normed_space F] {m : measurable_space α} {μ : measure_theory.measure α} (s t : set α) (hs : measurable_set s) (ht : measurable_set t) (hs_finite : μ s ) (ht_finite : μ t ) (h_inter : s t = ) :
theorem measure_theory.weighted_smul_smul {α : Type u_1} {F : Type u_3} {𝕜 : Type u_4} [normed_add_comm_group F] [normed_space F] {m : measurable_space α} {μ : measure_theory.measure α} [normed_field 𝕜] [normed_space 𝕜 F] [smul_comm_class 𝕜 F] (c : 𝕜) (s : set α) (x : F) :
theorem measure_theory.weighted_smul_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} (s : set α) (x : ) (hx : 0 x) :

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.

Bochner integral of simple functions whose codomain is a real normed_space. This is equal to ∑ x in f.range, (μ (f ⁻¹' {x})).to_real • x (see integral_eq).

Equations
theorem measure_theory.simple_func.integral_eq_sum_of_subset {α : Type u_1} {F : Type u_3} [normed_add_comm_group F] [normed_space F] {m : measurable_space α} {μ : measure_theory.measure α} [decidable_pred (λ (x : F), x 0)] {f : measure_theory.simple_func α F} {s : finset F} (hs : finset.filter (λ (x : F), x 0) f.range s) :
measure_theory.simple_func.integral μ f = s.sum (λ (x : F), (μ (f ⁻¹' {x})).to_real x)

The Bochner integral is equal to a sum over any set that includes f.range (except 0).

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 α →ₛ ℝ≥0∞. But since ℝ≥0∞ 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 α →ₛ ℝ≥0∞. But since ℝ≥0∞ is not a normed_space, we need some form of coercion.

Positive part of a simple function in L1 space.

Equations

The Bochner integral of L1 #

Define the Bochner integral on α →₁ₛ[μ] E by extension from the simple functions α →₁ₛ[μ] E, and prove basic properties of this integral.

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

Equations

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

Equations
noncomputable def measure_theory.L1.integral_clm' {α : Type u_1} {E : Type u_2} (𝕜 : Type u_4) [normed_add_comm_group E] {m : measurable_space α} {μ : measure_theory.measure α} [normed_space E] [nontrivially_normed_field 𝕜] [normed_space 𝕜 E] [smul_comm_class 𝕜 E] [complete_space E] :

The Bochner integral in L1 space as a continuous linear map.

Equations

The Bochner integral in L1 space as a continuous linear map over ℝ.

Equations
@[irreducible]
noncomputable def measure_theory.L1.integral {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] {m : measurable_space α} {μ : measure_theory.measure α} [normed_space E] [complete_space E] (f : (measure_theory.Lp E 1 μ)) :
E

The Bochner integral in L1 space

Equations

The Bochner integral on functions #

Define the Bochner integral on functions generally to be the L1 Bochner integral, for integrable functions, and 0 otherwise; prove its basic properties.

@[irreducible]
noncomputable def measure_theory.integral {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} (μ : measure_theory.measure α) (f : α E) :
E

The Bochner integral

Equations

In the notation for integrals, an expression like ∫ x, g ‖x‖ ∂μ will not be parsed correctly, and needs parentheses. We do not set the binding power of r to 0, because then ∫ x, f x = 0 will be parsed incorrectly.

theorem measure_theory.integral_undef {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f : α E} {m : measurable_space α} {μ : measure_theory.measure α} (h : ¬measure_theory.integrable f μ) :
(a : α), f a μ = 0
theorem measure_theory.integral_zero (α : Type u_1) (E : Type u_2) [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} :
(a : α), 0 μ = 0
theorem measure_theory.integrable_of_integral_eq_one {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (h : (x : α), f x μ = 1) :
theorem measure_theory.integral_add {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f g : α E} {m : measurable_space α} {μ : measure_theory.measure α} (hf : measure_theory.integrable f μ) (hg : measure_theory.integrable g μ) :
(a : α), f a + g a μ = (a : α), f a μ + (a : α), g a μ
theorem measure_theory.integral_add' {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f g : α E} {m : measurable_space α} {μ : measure_theory.measure α} (hf : measure_theory.integrable f μ) (hg : measure_theory.integrable g μ) :
(a : α), (f + g) a μ = (a : α), f a μ + (a : α), g a μ
theorem measure_theory.integral_finset_sum {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} (s : finset ι) {f : ι α E} (hf : (i : ι), i s measure_theory.integrable (f i) μ) :
(a : α), s.sum (λ (i : ι), f i a) μ = s.sum (λ (i : ι), (a : α), f i a μ)
theorem measure_theory.integral_neg {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} (f : α E) :
(a : α), -f a μ = - (a : α), f a μ
theorem measure_theory.integral_neg' {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} (f : α E) :
(a : α), (-f) a μ = - (a : α), f a μ
theorem measure_theory.integral_sub {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f g : α E} {m : measurable_space α} {μ : measure_theory.measure α} (hf : measure_theory.integrable f μ) (hg : measure_theory.integrable g μ) :
(a : α), f a - g a μ = (a : α), f a μ - (a : α), g a μ
theorem measure_theory.integral_sub' {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f g : α E} {m : measurable_space α} {μ : measure_theory.measure α} (hf : measure_theory.integrable f μ) (hg : measure_theory.integrable g μ) :
(a : α), (f - g) a μ = (a : α), f a μ - (a : α), g a μ
theorem measure_theory.integral_smul {α : Type u_1} {E : Type u_2} {𝕜 : Type u_4} [normed_add_comm_group E] [normed_space E] [complete_space E] [nontrivially_normed_field 𝕜] [normed_space 𝕜 E] [smul_comm_class 𝕜 E] {m : measurable_space α} {μ : measure_theory.measure α} (c : 𝕜) (f : α E) :
(a : α), c f a μ = c (a : α), f a μ
theorem measure_theory.integral_mul_left {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {L : Type u_2} [is_R_or_C L] (r : L) (f : α L) :
(a : α), r * f a μ = r * (a : α), f a μ
theorem measure_theory.integral_mul_right {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {L : Type u_2} [is_R_or_C L] (r : L) (f : α L) :
(a : α), f a * r μ = (a : α), f a μ * r
theorem measure_theory.integral_div {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {L : Type u_2} [is_R_or_C L] (r : L) (f : α L) :
(a : α), f a / r μ = (a : α), f a μ / r
theorem measure_theory.integral_congr_ae {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f g : α E} {m : measurable_space α} {μ : measure_theory.measure α} (h : f =ᵐ[μ] g) :
(a : α), f a μ = (a : α), g a μ
@[continuity]
theorem measure_theory.integral_eq_zero_of_ae {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {f : α E} (hf : f =ᵐ[μ] 0) :
(a : α), f a μ = 0
theorem measure_theory.has_finite_integral.tendsto_set_integral_nhds_zero {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} {f : α E} (hf : measure_theory.has_finite_integral f μ) {l : filter ι} {s : ι set α} (hs : filter.tendsto (μ s) l (nhds 0)) :
filter.tendsto (λ (i : ι), (x : α) in s i, f x μ) l (nhds 0)

If f has finite integral, then ∫ x in s, f x ∂μ is absolutely continuous in s: it tends to zero as μ s tends to zero.

theorem measure_theory.integrable.tendsto_set_integral_nhds_zero {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} {f : α E} (hf : measure_theory.integrable f μ) {l : filter ι} {s : ι set α} (hs : filter.tendsto (μ s) l (nhds 0)) :
filter.tendsto (λ (i : ι), (x : α) in s i, f x μ) l (nhds 0)

If f is integrable, then ∫ x in s, f x ∂μ is absolutely continuous in s: it tends to zero as μ s tends to zero.

theorem measure_theory.tendsto_integral_of_L1 {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} (f : α E) (hfi : measure_theory.integrable f μ) {F : ι α E} {l : filter ι} (hFi : ∀ᶠ (i : ι) in l, measure_theory.integrable (F i) μ) (hF : filter.tendsto (λ (i : ι), ∫⁻ (x : α), 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} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {F : α E} {f : α E} (bound : α ) (F_measurable : (n : ), measure_theory.ae_strongly_measurable (F n) μ) (bound_integrable : measure_theory.integrable bound μ) (h_bound : (n : ), ∀ᵐ (a : α) μ, F n a bound a) (h_lim : ∀ᵐ (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. We could weaken the condition bound_integrable to require has_finite_integral bound μ instead (i.e. not requiring that bound is measurable), but in all applications proving integrability is easier.

theorem measure_theory.tendsto_integral_filter_of_dominated_convergence {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} {l : filter ι} [l.is_countably_generated] {F : ι α E} {f : α E} (bound : α ) (hF_meas : ∀ᶠ (n : ι) in l, measure_theory.ae_strongly_measurable (F n) μ) (h_bound : ∀ᶠ (n : ι) in l, ∀ᵐ (a : α) μ, F n a bound a) (bound_integrable : measure_theory.integrable bound μ) (h_lim : ∀ᵐ (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.has_sum_integral_of_dominated_convergence {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} [countable ι] {F : ι α E} {f : α E} (bound : ι α ) (hF_meas : (n : ι), measure_theory.ae_strongly_measurable (F n) μ) (h_bound : (n : ι), ∀ᵐ (a : α) μ, F n a bound n a) (bound_summable : ∀ᵐ (a : α) μ, summable (λ (n : ι), bound n a)) (bound_integrable : measure_theory.integrable (λ (a : α), ∑' (n : ι), bound n a) μ) (h_lim : ∀ᵐ (a : α) μ, has_sum (λ (n : ι), F n a) (f a)) :
has_sum (λ (n : ι), (a : α), F n a μ) ( (a : α), f a μ)

Lebesgue dominated convergence theorem for series.

theorem measure_theory.continuous_within_at_of_dominated {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {X : Type u_5} [topological_space X] [topological_space.first_countable_topology X] {F : X α E} {x₀ : X} {bound : α } {s : set X} (hF_meas : ∀ᶠ (x : X) in nhds_within x₀ s, measure_theory.ae_strongly_measurable (F x) μ) (h_bound : ∀ᶠ (x : X) in nhds_within x₀ s, ∀ᵐ (a : α) μ, F x a bound a) (bound_integrable : measure_theory.integrable bound μ) (h_cont : ∀ᵐ (a : α) μ, continuous_within_at (λ (x : X), F x a) s x₀) :
continuous_within_at (λ (x : X), (a : α), F x a μ) s x₀
theorem measure_theory.continuous_at_of_dominated {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {X : Type u_5} [topological_space X] [topological_space.first_countable_topology X] {F : X α E} {x₀ : X} {bound : α } (hF_meas : ∀ᶠ (x : X) in nhds x₀, measure_theory.ae_strongly_measurable (F x) μ) (h_bound : ∀ᶠ (x : X) in nhds x₀, ∀ᵐ (a : α) μ, F x a bound a) (bound_integrable : measure_theory.integrable bound μ) (h_cont : ∀ᵐ (a : α) μ, continuous_at (λ (x : X), F x a) x₀) :
continuous_at (λ (x : X), (a : α), F x a μ) x₀
theorem measure_theory.continuous_on_of_dominated {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {X : Type u_5} [topological_space X] [topological_space.first_countable_topology X] {F : X α E} {bound : α } {s : set X} (hF_meas : (x : X), x s measure_theory.ae_strongly_measurable (F x) μ) (h_bound : (x : X), x s (∀ᵐ (a : α) μ, F x a bound a)) (bound_integrable : measure_theory.integrable bound μ) (h_cont : ∀ᵐ (a : α) μ, continuous_on (λ (x : X), F x a) s) :
continuous_on (λ (x : X), (a : α), F x a μ) s
theorem measure_theory.continuous_of_dominated {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {X : Type u_5} [topological_space X] [topological_space.first_countable_topology X] {F : X α E} {bound : α } (hF_meas : (x : X), measure_theory.ae_strongly_measurable (F x) μ) (h_bound : (x : X), ∀ᵐ (a : α) μ, F x a bound a) (bound_integrable : measure_theory.integrable bound μ) (h_cont : ∀ᵐ (a : α) μ, continuous (λ (x : X), F x a)) :
continuous (λ (x : X), (a : α), F x a μ)

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} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 ≤ᵐ[μ] f) (hfm : measure_theory.ae_strongly_measurable f μ) :
(a : α), f a μ = (∫⁻ (a : α), ennreal.of_real (f a) μ).to_real
theorem measure_theory.integral_eq_integral_pos_part_sub_integral_neg_part {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : measure_theory.integrable f μ) :
(a : α), f a μ = (a : α), ((f a).to_nnreal) μ - (a : α), ((-f a).to_nnreal) μ
theorem measure_theory.integral_nonneg_of_ae {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 ≤ᵐ[μ] f) :
0 (a : α), f a μ
theorem measure_theory.lintegral_coe_eq_integral {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} (f : α nnreal) (hfi : measure_theory.integrable (λ (x : α), (f x)) μ) :
∫⁻ (a : α), (f a) μ = ennreal.of_real ( (a : α), (f a) μ)
theorem measure_theory.of_real_integral_eq_lintegral_of_real {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hfi : measure_theory.integrable f μ) (f_nn : 0 ≤ᵐ[μ] f) :
ennreal.of_real ( (x : α), f x μ) = ∫⁻ (x : α), ennreal.of_real (f x) μ
theorem measure_theory.integral_to_real {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α ennreal} (hfm : ae_measurable f μ) (hf : ∀ᵐ (x : α) μ, f x < ) :
(a : α), (f a).to_real μ = (∫⁻ (a : α), f a μ).to_real
theorem measure_theory.lintegral_coe_le_coe_iff_integral_le {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α nnreal} (hfi : measure_theory.integrable (λ (x : α), (f x)) μ) {b : nnreal} :
∫⁻ (a : α), (f a) μ b (a : α), (f a) μ b
theorem measure_theory.integral_coe_le_of_lintegral_coe_le {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α nnreal} {b : nnreal} (h : ∫⁻ (a : α), (f a) μ b) :
(a : α), (f a) μ b
theorem measure_theory.integral_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 f) :
0 (a : α), f a μ
theorem measure_theory.integral_nonpos_of_ae {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : f ≤ᵐ[μ] 0) :
(a : α), f a μ 0
theorem measure_theory.integral_nonpos {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : f 0) :
(a : α), f a μ 0
theorem measure_theory.integral_eq_zero_iff_of_nonneg_ae {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 ≤ᵐ[μ] f) (hfi : measure_theory.integrable f μ) :
(x : α), f x μ = 0 f =ᵐ[μ] 0
theorem measure_theory.integral_eq_zero_iff_of_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 f) (hfi : measure_theory.integrable f μ) :
(x : α), f x μ = 0 f =ᵐ[μ] 0
theorem measure_theory.integral_pos_iff_support_of_nonneg_ae {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 ≤ᵐ[μ] f) (hfi : measure_theory.integrable f μ) :
0 < (x : α), f x μ 0 < μ (function.support f)
theorem measure_theory.integral_pos_iff_support_of_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } (hf : 0 f) (hfi : measure_theory.integrable f μ) :
0 < (x : α), f x μ 0 < μ (function.support f)
theorem measure_theory.mem_ℒp.snorm_eq_integral_rpow_norm {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {H : Type u_6} [normed_add_comm_group H] {f : α H} {p : ennreal} (hp1 : p 0) (hp2 : p ) (hf : measure_theory.mem_ℒp f p μ) :
theorem measure_theory.integral_mono_ae {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f g : α } (hf : measure_theory.integrable f μ) (hg : measure_theory.integrable g μ) (h : f ≤ᵐ[μ] g) :
(a : α), f a μ (a : α), g a μ
theorem measure_theory.integral_mono {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f g : α } (hf : measure_theory.integrable f μ) (hg : measure_theory.integrable g μ) (h : f g) :
(a : α), f a μ (a : α), g a μ
theorem measure_theory.integral_mono_of_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f g : α } (hf : 0 ≤ᵐ[μ] f) (hgi : measure_theory.integrable g μ) (h : f ≤ᵐ[μ] g) :
(a : α), f a μ (a : α), g a μ
theorem measure_theory.integral_mono_measure {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {f : α } {ν : measure_theory.measure α} (hle : μ ν) (hf : 0 ≤ᵐ[ν] f) (hfi : measure_theory.integrable f ν) :
(a : α), f a μ (a : α), f a ν
theorem measure_theory.norm_integral_le_integral_norm {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} (f : α E) :
(a : α), f a μ (a : α), f a μ
theorem measure_theory.norm_integral_le_of_norm_le {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {f : α E} {g : α } (hg : measure_theory.integrable g μ) (h : ∀ᵐ (x : α) μ, f x g x) :
(x : α), f x μ (x : α), g x μ
@[simp]
theorem measure_theory.integral_const {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} (c : E) :
(x : α), c μ = (μ set.univ).to_real c
theorem measure_theory.tendsto_integral_approx_on_of_measurable {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} [measurable_space E] [borel_space E] {f : α E} {s : set E} [topological_space.separable_space s] (hfi : measure_theory.integrable f μ) (hfm : measurable f) (hs : ∀ᵐ (x : α) μ, f x closure s) {y₀ : E} (h₀ : y₀ s) (h₀i : measure_theory.integrable (λ (x : α), y₀) μ) :
theorem measure_theory.integral_add_measure {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ ν : measure_theory.measure α} {f : α E} (hμ : measure_theory.integrable f μ) (hν : measure_theory.integrable f ν) :
(x : α), f x + ν) = (x : α), f x μ + (x : α), f x ν
@[simp]
theorem measure_theory.integral_zero_measure {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} (f : α E) :
(x : α), f x 0 = 0
theorem measure_theory.integral_finset_sum_measure {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {ι : Type u_3} {m : measurable_space α} {f : α E} {μ : ι measure_theory.measure α} {s : finset ι} (hf : (i : ι), i s measure_theory.integrable f (μ i)) :
(a : α), f a s.sum (λ (i : ι), μ i) = s.sum (λ (i : ι), (a : α), f a μ i)
theorem measure_theory.nndist_integral_add_measure_le_lintegral {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {f : α E} {m : measurable_space α} {μ ν : measure_theory.measure α} (h₁ : measure_theory.integrable f μ) (h₂ : measure_theory.integrable f ν) :
(has_nndist.nndist ( (x : α), f x μ) ( (x : α), f x + ν))) ∫⁻ (x : α), f x‖₊ ν
theorem measure_theory.has_sum_integral_measure {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {ι : Type u_3} {m : measurable_space α} {f : α E} {μ : ι measure_theory.measure α} (hf : measure_theory.integrable f (measure_theory.measure.sum μ)) :
has_sum (λ (i : ι), (a : α), f a μ i) ( (a : α), f a measure_theory.measure.sum μ)
theorem measure_theory.integral_sum_measure {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {ι : Type u_3} {m : measurable_space α} {f : α E} {μ : ι measure_theory.measure α} (hf : measure_theory.integrable f (measure_theory.measure.sum μ)) :
(a : α), f a measure_theory.measure.sum μ = ∑' (i : ι), (a : α), f a μ i
theorem measure_theory.integral_tsum {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {ι : Type u_3} [countable ι] {f : ι α E} (hf : (i : ι), measure_theory.ae_strongly_measurable (f i) μ) (hf' : ∑' (i : ι), ∫⁻ (a : α), f i a‖₊ μ ) :
(a : α), ∑' (i : ι), f i a μ = ∑' (i : ι), (a : α), f i a μ
@[simp]
theorem measure_theory.integral_smul_measure {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} (f : α E) (c : ennreal) :
(x : α), f x c μ = c.to_real (x : α), f x μ
theorem measure_theory.integral_map_of_strongly_measurable {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_3} [measurable_space β] {φ : α β} (hφ : measurable φ) {f : β E} (hfm : measure_theory.strongly_measurable f) :
(y : β), f y measure_theory.measure.map φ μ = (x : α), f (φ x) μ
theorem measure_theory.integral_map {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_3} [measurable_space β] {φ : α β} (hφ : ae_measurable φ μ) {f : β E} (hfm : measure_theory.ae_strongly_measurable f (measure_theory.measure.map φ μ)) :
(y : β), f y measure_theory.measure.map φ μ = (x : α), f (φ x) μ
theorem measurable_embedding.integral_map {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_3} {_x : measurable_space β} {f : α β} (hf : measurable_embedding f) (g : β E) :
(y : β), g y measure_theory.measure.map f μ = (x : α), g (f x) μ
theorem closed_embedding.integral_map {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_3} [topological_space α] [borel_space α] [topological_space β] [measurable_space β] [borel_space β] {φ : α β} (hφ : closed_embedding φ) (f : β E) :
(y : β), f y measure_theory.measure.map φ μ = (x : α), f (φ x) μ
theorem measure_theory.integral_map_equiv {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_3} [measurable_space β] (e : α ≃ᵐ β) (f : β E) :
(y : β), f y measure_theory.measure.map e μ = (x : α), f (e x) μ
theorem measure_theory.measure_preserving.integral_comp {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {m : measurable_space α} {μ : measure_theory.measure α} {β : Type u_3} {_x : measurable_space β} {f : α β} {ν : measure_theory.measure β . "volume_tac"} (h₁ : measure_theory.measure_preserving f μ ν) (h₂ : measurable_embedding f) (g : β E) :
(x : α), g (f x) μ = (y : β), g y ν
theorem measure_theory.set_integral_eq_subtype {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {α : Type u_1} [measure_theory.measure_space α] {s : set α} (hs : measurable_set s) (f : α E) :
(x : α) in s, f x = (x : s), f x
@[simp]
theorem measure_theory.set_integral_dirac' {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] {mα : measurable_space α} {f : α E} (hf : measure_theory.strongly_measurable f) (a : α) {s : set α} (hs : measurable_set s) [decidable (a s)] :
(x : α) in s, f x measure_theory.measure.dirac a = ite (a s) (f a) 0
theorem measure_theory.set_integral_dirac {α : Type u_1} {E : Type u_2} [normed_add_comm_group E] [normed_space E] [complete_space E] [measurable_space α] [measurable_singleton_class α] (f : α E) (a : α) (s : set α) [decidable (a s)] :
(x : α) in s, f x measure_theory.measure.dirac a = ite (a s) (f a) 0
theorem measure_theory.mul_meas_ge_le_integral_of_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} [measure_theory.is_finite_measure μ] {f : α } (hf_nonneg : 0 f) (hf_int : measure_theory.integrable f μ) (ε : ) :
ε * (μ {x : α | ε f x}).to_real (x : α), f x μ
theorem measure_theory.integral_mul_norm_le_Lp_mul_Lq {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {E : Type u_2} [normed_add_comm_group E] {f g : α E} {p q : } (hpq : p.is_conjugate_exponent q) (hf : measure_theory.mem_ℒp f (ennreal.of_real p) μ) (hg : measure_theory.mem_ℒp g (ennreal.of_real q) μ) :
(a : α), f a * g a μ ( (a : α), f a ^ p μ) ^ (1 / p) * ( (a : α), g a ^ q μ) ^ (1 / q)

Hölder's inequality for the integral of a product of norms. The integral of the product of two norms of functions is bounded by the product of their ℒp and ℒq seminorms when p and q are conjugate exponents.

theorem measure_theory.integral_mul_le_Lp_mul_Lq_of_nonneg {α : Type u_1} {m : measurable_space α} {μ : measure_theory.measure α} {p q : } (hpq : p.is_conjugate_exponent q) {f g : α } (hf_nonneg : 0 ≤ᵐ[μ] f) (hg_nonneg : 0 ≤ᵐ[μ] g) (hf : measure_theory.mem_ℒp f (ennreal.of_real p) μ) (hg : measure_theory.mem_ℒp g (ennreal.of_real q) μ) :
(a : α), f a * g a μ ( (a : α), f a ^ p μ) ^ (1 / p) * ( (a : α), g a ^ q μ) ^ (1 / q)

Hölder's inequality for functions α → ℝ. The integral of the product of two nonnegative functions is bounded by the product of their ℒp and ℒq seminorms when p and q are conjugate exponents.

Simple function seen as simple function of a larger measurable_space.

Equations
theorem measure_theory.integral_simple_func_larger_space {F : Type u_3} [normed_add_comm_group F] [normed_space F] [complete_space F] {β : Type u_6} {m m0 : measurable_space β} {μ : measure_theory.measure β} (hm : m m0) (f : measure_theory.simple_func β F) (hf_int : measure_theory.integrable f μ) :
(x : β), f x μ = f.range.sum (λ (x : F), (μ (f ⁻¹' {x})).to_real x)
theorem measure_theory.integral_trim_simple_func {F : Type u_3} [normed_add_comm_group F] [normed_space F] [complete_space F] {β : Type u_6} {m m0 : measurable_space β} {μ : measure_theory.measure β} (hm : m m0) (f : measure_theory.simple_func β F) (hf_int : measure_theory.integrable f μ) :
(x : β), f x μ = (x : β), f x μ.trim hm
theorem measure_theory.integral_trim {F : Type u_3} [normed_add_comm_group F] [normed_space F] [complete_space F] {β : Type u_6} {m m0 : measurable_space β} {μ : measure_theory.measure β} (hm : m m0) {f : β F} (hf : measure_theory.strongly_measurable f) :
(x : β), f x μ = (x : β), f x μ.trim hm
theorem measure_theory.integral_trim_ae {F : Type u_3} [normed_add_comm_group F] [normed_space F] [complete_space F] {β : Type u_6} {m m0 : measurable_space β} {μ : measure_theory.measure β} (hm : m m0) {f : β F} (hf : measure_theory.ae_strongly_measurable f (μ.trim hm)) :
(x : β), f x μ = (x : β), f x μ.trim hm
theorem measure_theory.snorm_one_le_of_le {α : Type u_1} {m0 : measurable_space α} {μ : measure_theory.measure α} {r : nnreal} {f : α } (hfint : measure_theory.integrable f μ) (hfint' : 0 (x : α), f x μ) (hf : ∀ᵐ (ω : α) μ, f ω r) :
theorem measure_theory.snorm_one_le_of_le' {α : Type u_1} {m0 : measurable_space α} {μ : measure_theory.measure α} {r : } {f : α } (hfint : measure_theory.integrable f μ) (hfint' : 0 (x : α), f x μ) (hf : ∀ᵐ (ω : α) μ, f ω r) :