Integrable functions and L¹ space #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In the first part of this file, the predicate integrable is defined and basic properties of
integrable functions are proved.
Such a predicate is already available under the name mem_ℒp 1. We give a direct definition which
is easier to use, and show that it is equivalent to mem_ℒp 1
In the second part, we establish an API between integrable and the space L¹ of equivalence
classes of integrable functions, already defined as a special case of L^p spaces for p = 1.
Notation #
-
α →₁[μ] βis the type ofL¹space, whereαis ameasure_spaceandβis anormed_add_comm_groupwith asecond_countable_topology.f : α →ₘ βis a "function" inL¹. In comments,[f]is also used to denote anL¹function.₁can be typed as\1.
Main definitions #
-
Let
f : α → βbe a function, whereαis ameasure_spaceandβanormed_add_comm_group. Thenhas_finite_integral fmeans(∫⁻ a, ‖f a‖₊) < ∞. -
If
βis moreover ameasurable_spacethenfis calledintegrableiffismeasurableandhas_finite_integral fholds.
Implementation notes #
To prove something for an arbitrary integrable function, a useful theorem is
integrable.induction in the file set_integral.
Tags #
integrable, function space, l1
Some results about the Lebesgue integral involving a normed group #
The predicate has_finite_integral #
has_finite_integral f μ means that the integral ∫⁻ a, ‖f a‖ ∂μ is finite.
has_finite_integral f means has_finite_integral f volume.
Lemmas used for defining the positive part of a L¹ function
The predicate integrable #
integrable f μ means that f is measurable and that the integral ∫⁻ a, ‖f a‖ ∂μ is finite.
integrable f means integrable f volume.
Equations
Hölder's inequality for integrable functions: the scalar multiplication of an integrable vector-valued function by a scalar function with finite essential supremum is integrable.
Hölder's inequality for integrable functions: the scalar multiplication of an integrable scalar-valued function by a vector-value function with finite essential supremum is integrable.
A non-quantitative version of Markov inequality for integrable functions: the measure of points
where ‖f x‖ ≥ ε is finite for all positive ε.
The map u ↦ f • u is an isometry between the L^1 spaces for μ.with_density f and μ.
Equations
- measure_theory.with_density_smul_li μ f_meas = {to_linear_map := {to_fun := λ (u : ↥(measure_theory.Lp E 1 (μ.with_density (λ (x : α), ↑(f x))))), measure_theory.mem_ℒp.to_Lp (λ (x : α), f x • ⇑u x) _, map_add' := _, map_smul' := _}, norm_map' := _}
Lemmas used for defining the positive part of a L¹ function #
The predicate integrable on measurable functions modulo a.e.-equality #
A class of almost everywhere equal functions is integrable if its function representative
is integrable.
Equations
Computing the norm of a difference between two L¹-functions. Note that this is not a
special case of norm_def since (f - g) x and f x - g x are not equal
(but only a.e.-equal).
Computing the norm of a difference between two L¹-functions. Note that this is not a
special case of of_real_norm_eq_lintegral since (f - g) x and f x - g x are not equal
(but only a.e.-equal).
Construct the equivalence class [f] of an integrable function f, as a member of the
space L1 β 1 μ.