Lp space #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file provides the space Lp E p μ
as the subtype of elements of α →ₘ[μ] E
(see ae_eq_fun)
such that snorm f p μ
is finite. For 1 ≤ p
, snorm
defines a norm and Lp
is a complete metric
space.
Main definitions #
Lp E p μ
: elements ofα →ₘ[μ] E
(see ae_eq_fun) such thatsnorm f p μ
is finite. Defined as anadd_subgroup
ofα →ₘ[μ] E
.
Lipschitz functions vanishing at zero act by composition on Lp
. We define this action, and prove
that it is continuous. In particular,
continuous_linear_map.comp_Lp
defines the action onLp
of a continuous linear map.Lp.pos_part
is the positive part of anLp
function.Lp.neg_part
is the negative part of anLp
function.
When α
is a topological space equipped with a finite Borel measure, there is a bounded linear map
from the normed space of bounded continuous functions (α →ᵇ E
) to Lp E p μ
. We construct this
as bounded_continuous_function.to_Lp
.
Notations #
α →₁[μ] E
: the typeLp E 1 μ
.α →₂[μ] E
: the typeLp E 2 μ
.
Implementation #
Since Lp
is defined as an add_subgroup
, dot notation does not work. Use Lp.measurable f
to
say that the coercion of f
to a genuine function is measurable, instead of the non-working
f.measurable
.
To prove that two Lp
elements are equal, it suffices to show that their coercions to functions
coincide almost everywhere (this is registered as an ext
rule). This can often be done using
filter_upwards
. For instance, a proof from first principles that f + (g + h) = (f + g) + h
could read (in the Lp
namespace)
example (f g h : Lp E p μ) : (f + g) + h = f + (g + h) :=
begin
ext1,
filter_upwards [coe_fn_add (f + g) h, coe_fn_add f g, coe_fn_add f (g + h), coe_fn_add g h]
with _ ha1 ha2 ha3 ha4,
simp only [ha1, ha2, ha3, ha4, add_assoc],
end
The lemma coe_fn_add
states that the coercion of f + g
coincides almost everywhere with the sum
of the coercions of f
and g
. All such lemmas use coe_fn
in their name, to distinguish the
function coercion from the coercion to almost everywhere defined functions.
Lp space #
The space of equivalence classes of measurable functions for which snorm f p μ < ∞
.
Lp space
Equations
Instances for ↥measure_theory.Lp
- measure_theory.Lp.has_coe_to_fun
- measure_theory.Lp.has_norm
- measure_theory.Lp.has_nnnorm
- measure_theory.Lp.has_dist
- measure_theory.Lp.has_edist
- measure_theory.Lp.normed_add_comm_group
- measure_theory.Lp.module
- measure_theory.Lp.is_central_scalar
- measure_theory.Lp.smul_comm_class
- measure_theory.Lp.is_scalar_tower
- measure_theory.Lp.has_bounded_smul
- measure_theory.Lp.normed_space
- measure_theory.Lp.complete_space
- measure_theory.Lp.has_le.le.covariant_class
- measure_theory.Lp.ordered_add_comm_group
- measure_theory.Lp.lattice
- measure_theory.Lp.normed_lattice_add_comm_group
- measure_theory.L2.measure_theory.Lp.has_inner
- measure_theory.L2.inner_product_space
make an element of Lp from a function verifying mem_ℒp
Equations
- measure_theory.mem_ℒp.to_Lp f h_mem_ℒp = ⟨measure_theory.ae_eq_fun.mk f _, _⟩
Equations
- measure_theory.Lp.has_coe_to_fun = {coe := λ (f : ↥(measure_theory.Lp E p μ)), ⇑↑f}
Equations
- measure_theory.Lp.has_norm = {norm := λ (f : ↥(measure_theory.Lp E p μ)), (measure_theory.snorm ⇑f p μ).to_real}
Equations
- measure_theory.Lp.has_nnnorm = {nnnorm := λ (f : ↥(measure_theory.Lp E p μ)), ⟨‖f‖, _⟩}
Equations
- measure_theory.Lp.has_dist = {dist := λ (f g : ↥(measure_theory.Lp E p μ)), ‖f - g‖}
Equations
- measure_theory.Lp.has_edist = {edist := λ (f g : ↥(measure_theory.Lp E p μ)), measure_theory.snorm (⇑f - ⇑g) p μ}
Equations
- measure_theory.Lp.normed_add_comm_group = {to_has_norm := normed_add_comm_group.to_has_norm {to_fun := has_norm.norm measure_theory.Lp.has_norm, map_zero' := _, add_le' := _, neg' := _, eq_zero_of_map_eq_zero' := _}.to_normed_add_comm_group, to_add_comm_group := normed_add_comm_group.to_add_comm_group {to_fun := has_norm.norm measure_theory.Lp.has_norm, map_zero' := _, add_le' := _, neg' := _, eq_zero_of_map_eq_zero' := _}.to_normed_add_comm_group, to_metric_space := {to_pseudo_metric_space := {to_has_dist := pseudo_metric_space.to_has_dist metric_space.to_pseudo_metric_space, dist_self := _, dist_comm := _, dist_triangle := _, edist := has_edist.edist measure_theory.Lp.has_edist, edist_dist := _, to_uniform_space := pseudo_metric_space.to_uniform_space metric_space.to_pseudo_metric_space, uniformity_dist := _, to_bornology := pseudo_metric_space.to_bornology metric_space.to_pseudo_metric_space, cobounded_sets := _}, eq_of_dist_eq_zero := _}, dist_eq := _}
The 𝕜
-submodule of elements of α →ₘ[μ] E
whose Lp
norm is finite. This is Lp E p μ
,
with extra structure.
Equations
- measure_theory.Lp.Lp_submodule E p μ 𝕜 = {carrier := (measure_theory.Lp E p μ).carrier, add_mem' := _, zero_mem' := _, smul_mem' := _}
Equations
- measure_theory.Lp.module = {to_distrib_mul_action := module.to_distrib_mul_action (measure_theory.Lp.Lp_submodule E p μ 𝕜).module, add_smul := _, zero_smul := _}
Equations
- measure_theory.Lp.normed_space = {to_module := measure_theory.Lp.module measure_theory.Lp.normed_space._proof_1, norm_smul_le := _}
Indicator of a set as an element of Lᵖ #
For a set s
with (hs : measurable_set s)
and (hμs : μ s < ∞)
, we build
indicator_const_Lp p hs hμs c
, the element of Lp
corresponding to s.indicator (λ x, c)
.
The ℒ^p
norm of the indicator of a set is uniformly small if the set itself has small measure,
for any p < ∞
. Given here as an existential ∀ ε > 0, ∃ η > 0, ...
to avoid later
management of ℝ≥0∞
-arithmetic.
Indicator of a set as an element of Lp
.
Equations
- measure_theory.indicator_const_Lp p hs hμs c = measure_theory.mem_ℒp.to_Lp (s.indicator (λ (_x : α), c)) _
The indicator of a disjoint union of two sets is the sum of the indicators of the sets.
Composition on L^p
#
We show that Lipschitz functions vanishing at zero act by composition on L^p
, and specialize
this to the composition with continuous linear maps, and to the definition of the positive
part of an L^p
function.
When g
is a Lipschitz function sending 0
to 0
and f
is in Lp
, then g ∘ f
is well
defined as an element of Lp
.
Equations
- hg.comp_Lp g0 f = ⟨measure_theory.ae_eq_fun.comp g _ ↑f, _⟩
Composing f : Lp
with L : E →L[𝕜] F
.
Composing f : Lp E p μ
with L : E →L[𝕜] F
, seen as a 𝕜
-linear map on Lp E p μ
.
Equations
- continuous_linear_map.comp_Lpₗ p μ L = {to_fun := λ (f : ↥(measure_theory.Lp E p μ)), L.comp_Lp f, map_add' := _, map_smul' := _}
Composing f : Lp E p μ
with L : E →L[𝕜] F
, seen as a continuous 𝕜
-linear map on
Lp E p μ
. See also the similar
linear_map.comp_left
for functions,continuous_linear_map.comp_left_continuous
for continuous functions,continuous_linear_map.comp_left_continuous_bounded
for bounded continuous functions,continuous_linear_map.comp_left_continuous_compact
for continuous functions on compact spaces.
Equations
- continuous_linear_map.comp_LpL p μ L = (continuous_linear_map.comp_Lpₗ p μ L).mk_continuous ‖L‖ _
Positive part of a function in L^p
.
Equations
- measure_theory.Lp.pos_part f = measure_theory.Lp.lipschitz_with_pos_part.comp_Lp measure_theory.Lp.pos_part._proof_1 f
Negative part of a function in L^p
.
Equations
L^p
is a complete space #
We show that L^p
is a complete space for 1 ≤ p
.
Lp
is complete iff Cauchy sequences of ℒp
have limits in ℒp
#
Prove that controlled Cauchy sequences of ℒp
have limits in ℒp
#
Lp
is complete for 1 ≤ p
#
Continuous functions in Lp
#
An additive subgroup of Lp E p μ
, consisting of the equivalence classes which contain a
bounded continuous representative.
By definition, the elements of Lp.bounded_continuous_function E p μ
are the elements of
Lp E p μ
which contain a bounded continuous representative.
A bounded continuous function on a finite-measure space is in Lp
.
The Lp
-norm of a bounded continuous function is at most a constant (depending on the measure
of the whole space) times its sup-norm.
The Lp
-norm of a bounded continuous function is at most a constant (depending on the measure
of the whole space) times its sup-norm.
The normed group homomorphism of considering a bounded continuous function on a finite-measure
space as an element of Lp
.
Equations
The bounded linear map of considering a bounded continuous function on a finite-measure space
as an element of Lp
.
Equations
- bounded_continuous_function.to_Lp p μ 𝕜 = (linear_map.cod_restrict (measure_theory.Lp.Lp_submodule E p μ 𝕜) ((continuous_map.to_ae_eq_fun_linear_map μ).comp (bounded_continuous_function.to_continuous_map_linear_map α E 𝕜)) bounded_continuous_function.mem_Lp).mk_continuous (↑(measure_theory.measure_univ_nnreal μ) ^ (p.to_real)⁻¹) bounded_continuous_function.Lp_norm_le
The bounded linear map of considering a continuous function on a compact finite-measure
space α
as an element of Lp
. By definition, the norm on C(α, E)
is the sup-norm, transferred
from the space α →ᵇ E
of bounded continuous functions, so this construction is just a matter of
transferring the structure from bounded_continuous_function.to_Lp
along the isometry.
Equations
If a sum of continuous functions g n
is convergent, and the same sum converges in Lᵖ
to h
,
then in fact g n
converges uniformly to h
.
Bound for the operator norm of continuous_map.to_Lp
.
A version of Markov's inequality with elements of Lp.