Equivalences among $L^p$ spaces #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we collect a variety of equivalences among various $L^p$ spaces. In particular,
when α
is a fintype
, given E : α → Type u
and p : ℝ≥0∞
, there is a natural linear isometric
equivalence lp_pi_Lpₗᵢ : lp E p ≃ₗᵢ pi_Lp p E
. In addition, when α
is a discrete topological
space, the bounded continuous functions α →ᵇ β
correspond exactly to lp (λ _, β) ∞
. Here there
can be more structure, including ring and algebra structures, and we implement these equivalences
accordingly as well.
We keep this as a separate file so that the various $L^p$ space files don't import the others.
Recall that pi_Lp
is just a type synonym for Π i, E i
but given a different metric and norm
structure, although the topological, uniform and bornological structures coincide definitionally.
These structures are only defined on pi_Lp
for fintype α
, so there are no issues of convergence
to consider.
While pre_lp
is also a type synonym for Π i, E i
, it allows for infinite index types. On this
type there is a predicate mem_ℓp
which says that the relevant p
-norm is finite and lp E p
is
the subtype of pre_lp
satisfying mem_ℓp
.
TODO #
- Equivalence between
lp
andmeasure_theory.Lp
, forf : α → E
(i.e., functions rather than pi-types) and the counting measure onα
The canonical add_equiv
between lp E p
and pi_Lp p E
when E : α → Type u
with
[fintype α]
and [fact (1 ≤ p)]
.
Equations
- add_equiv.lp_pi_Lp = {to_fun := equiv.lp_pi_Lp.to_fun, inv_fun := equiv.lp_pi_Lp.inv_fun, left_inv := _, right_inv := _, map_add' := _}
The canonical linear_isometry_equiv
between lp E p
and pi_Lp p E
when E : α → Type u
with [fintype α]
and [fact (1 ≤ p)]
.
Equations
- lp_pi_Lpₗᵢ 𝕜 = {to_linear_equiv := {to_fun := add_equiv.lp_pi_Lp.to_fun, map_add' := _, map_smul' := _, inv_fun := add_equiv.lp_pi_Lp.inv_fun, left_inv := _, right_inv := _}, norm_map' := _}
The canonical map between lp (λ (_ : α), E) ∞
and α →ᵇ E
as an add_equiv
.
The canonical map between lp (λ (_ : α), E) ∞
and α →ᵇ E
as a linear_isometry_equiv
.
The canonical map between lp (λ (_ : α), R) ∞
and α →ᵇ R
as a ring_equiv
.
Equations
- ring_equiv.lp_bcf R = {to_fun := add_equiv.lp_bcf.to_fun, inv_fun := add_equiv.lp_bcf.inv_fun, left_inv := _, right_inv := _, map_mul' := _, map_add' := _}
The canonical map between lp (λ (_ : α), A) ∞
and α →ᵇ A
as an alg_equiv
.
Equations
- alg_equiv.lp_bcf α A 𝕜 = {to_fun := (ring_equiv.lp_bcf A).to_fun, inv_fun := (ring_equiv.lp_bcf A).inv_fun, left_inv := _, right_inv := _, map_mul' := _, map_add' := _, commutes' := _}