Functions a.e. measurable with respect to a sub-σ-algebra #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
A function f verifies ae_strongly_measurable' m f μ if it is μ-a.e. equal to
an m-strongly measurable function. This is similar to ae_strongly_measurable, but the
measurable_space structures used for the measurability statement and for the measure are
different.
We define Lp_meas F 𝕜 m p μ, the subspace of Lp F p μ containing functions f verifying
ae_strongly_measurable' m f μ, i.e. functions which are μ-a.e. equal to an m-strongly
measurable function.
Main statements #
We define an isometry_equiv between Lp_meas_subgroup and the Lp space corresponding to the
measure μ.trim hm. As a consequence, the completeness of Lp implies completeness of Lp_meas.
Lp.induction_strongly_measurable (see also mem_ℒp.induction_strongly_measurable):
To prove something for an Lp function a.e. strongly measurable with respect to a
sub-σ-algebra m in a normed space, it suffices to show that
- the property holds for (multiples of) characteristic functions which are measurable w.r.t.
m; - is closed under addition;
- the set of functions in
Lpstrongly measurable w.r.t.mfor which the property holds is closed.
A function f verifies ae_strongly_measurable' m f μ if it is μ-a.e. equal to
an m-strongly measurable function. This is similar to ae_strongly_measurable, but the
measurable_space structures used for the measurability statement and for the measure are
different.
Equations
- measure_theory.ae_strongly_measurable' m f μ = ∃ (g : α → β), measure_theory.strongly_measurable g ∧ f =ᵐ[μ] g
An m-strongly measurable function almost everywhere equal to f.
Equations
If the restriction to a set s of a σ-algebra m is included in the restriction to s of
another σ-algebra m₂ (hypothesis hs), the set s is m measurable and a function f almost
everywhere supported on s is m-ae-strongly-measurable, then f is also
m₂-ae-strongly-measurable.
The subset Lp_meas of Lp functions a.e. measurable with respect to a sub-sigma-algebra #
Lp_meas_subgroup F m p μ is the subspace of Lp F p μ containing functions f verifying
ae_strongly_measurable' m f μ, i.e. functions which are μ-a.e. equal to
an m-strongly measurable function.
Equations
- measure_theory.Lp_meas_subgroup F m p μ = {carrier := {f : ↥(measure_theory.Lp F p μ) | measure_theory.ae_strongly_measurable' m ⇑f μ}, add_mem' := _, zero_mem' := _, neg_mem' := _}
Instances for ↥measure_theory.Lp_meas_subgroup
Lp_meas F 𝕜 m p μ is the subspace of Lp F p μ containing functions f verifying
ae_strongly_measurable' m f μ, i.e. functions which are μ-a.e. equal to
an m-strongly measurable function.
Equations
- measure_theory.Lp_meas F 𝕜 m p μ = {carrier := {f : ↥(measure_theory.Lp F p μ) | measure_theory.ae_strongly_measurable' m ⇑f μ}, add_mem' := _, zero_mem' := _, smul_mem' := _}
Instances for ↥measure_theory.Lp_meas
The subspace Lp_meas is complete. #
We define an isometry_equiv between Lp_meas_subgroup and the Lp space corresponding to the
measure μ.trim hm. As a consequence, the completeness of Lp implies completeness of
Lp_meas_subgroup (and Lp_meas).
If f belongs to Lp_meas_subgroup F m p μ, then the measurable function it is almost
everywhere equal to (given by ae_measurable.mk) belongs to ℒp for the measure μ.trim hm.
If f belongs to Lp for the measure μ.trim hm, then it belongs to the subgroup
Lp_meas_subgroup F m p μ.
Map from Lp_meas_subgroup to Lp F p (μ.trim hm).
Equations
Map from Lp_meas to Lp F p (μ.trim hm).
Equations
- measure_theory.Lp_meas_to_Lp_trim F 𝕜 p μ hm f = measure_theory.mem_ℒp.to_Lp (Exists.some _) _
Map from Lp F p (μ.trim hm) to Lp_meas_subgroup, inverse of
Lp_meas_subgroup_to_Lp_trim.
Equations
- measure_theory.Lp_trim_to_Lp_meas_subgroup F p μ hm f = ⟨measure_theory.mem_ℒp.to_Lp ⇑f _, _⟩
Map from Lp F p (μ.trim hm) to Lp_meas, inverse of Lp_meas_to_Lp_trim.
Equations
- measure_theory.Lp_trim_to_Lp_meas F 𝕜 p μ hm f = ⟨measure_theory.mem_ℒp.to_Lp ⇑f _, _⟩
Lp_trim_to_Lp_meas_subgroup is a right inverse of Lp_meas_subgroup_to_Lp_trim.
Lp_trim_to_Lp_meas_subgroup is a left inverse of Lp_meas_subgroup_to_Lp_trim.
Lp_meas_subgroup_to_Lp_trim preserves the norm.
Lp_meas_subgroup and Lp F p (μ.trim hm) are isometric.
Equations
- measure_theory.Lp_meas_subgroup_to_Lp_trim_iso F p μ hm = {to_equiv := {to_fun := measure_theory.Lp_meas_subgroup_to_Lp_trim F p μ hm, inv_fun := measure_theory.Lp_trim_to_Lp_meas_subgroup F p μ hm, left_inv := _, right_inv := _}, isometry_to_fun := _}
Lp_meas_subgroup and Lp_meas are isometric.
Equations
Lp_meas and Lp F p (μ.trim hm) are isometric, with a linear equivalence.
Equations
- measure_theory.Lp_meas_to_Lp_trim_lie F 𝕜 p μ hm = {to_linear_equiv := {to_fun := measure_theory.Lp_meas_to_Lp_trim F 𝕜 p μ hm, map_add' := _, map_smul' := _, inv_fun := measure_theory.Lp_trim_to_Lp_meas F 𝕜 p μ hm, left_inv := _, right_inv := _}, norm_map' := _}
We do not get ae_fin_strongly_measurable f (μ.trim hm), since we don't have
f =ᵐ[μ.trim hm] Lp_meas_to_Lp_trim F 𝕜 p μ hm f but only the weaker
f =ᵐ[μ] Lp_meas_to_Lp_trim F 𝕜 p μ hm f.
When applying the inverse of Lp_meas_to_Lp_trim_lie (which takes a function in the Lp space of
the sub-sigma algebra and returns its version in the larger Lp space) to an indicator of the
sub-sigma-algebra, we obtain an indicator in the Lp space of the larger sigma-algebra.
Auxiliary lemma for Lp.induction_strongly_measurable.
To prove something for an Lp function a.e. strongly measurable with respect to a
sub-σ-algebra m in a normed space, it suffices to show that
- the property holds for (multiples of) characteristic functions which are measurable w.r.t.
m; - is closed under addition;
- the set of functions in
Lpstrongly measurable w.r.t.mfor which the property holds is closed.
To prove something for an arbitrary mem_ℒp function a.e. strongly measurable with respect
to a sub-σ-algebra m in a normed space, it suffices to show that
- the property holds for (multiples of) characteristic functions which are measurable w.r.t.
m; - is closed under addition;
- the set of functions in the
Lᵖspace strongly measurable w.r.t.mfor which the property holds is closed. - the property is closed under the almost-everywhere equal relation.