ℓp space #
This file describes properties of elements f of a pi-type Π i, E i with finite "norm",
defined for p:ℝ≥0∞ as the size of the support of f if p=0, (∑' a, ∥f a∥^p) ^ (1/p) for
0 < p < ∞ and ⨆ a, ∥f a∥ for p=∞.
The Prop-valued mem_ℓp f p states that a function f : Π i, E i has finite norm according
to the above definition; that is, f has finite support if p = 0, summable (λ a, ∥f a∥^p) if
0 < p < ∞, and bdd_above (norm '' (set.range f)) if p = ∞.
The space lp E p is the subtype of elements of Π i : α, E i which satisfy mem_ℓp f p. For
1 ≤ p, the "norm" is genuinely a norm and lp is a complete metric space.
Main definitions #
mem_ℓp f p: property that the functionfsatisfies, as appropriate,ffinitely supported ifp = 0,summable (λ a, ∥f a∥^p)if0 < p < ∞, andbdd_above (norm '' (set.range f))ifp = ∞lp E p: elements ofΠ i : α, E isuch thatmem_ℓp f p. Defined as anadd_subgroupof a type synonympre_lpforΠ i : α, E i, and equipped with anormed_groupstructure; also equipped withnormed_space 𝕜andcomplete_spaceinstances under appropriate conditions
Main results #
mem_ℓp.of_exponent_ge: Forq ≤ p, a function which ismem_ℓpforqis alsomem_ℓpforplp.mem_ℓp_of_tendsto,lp.norm_le_of_tendsto: A pointwise limit of functions inlp, all withlpnorm≤ C, is itself inlpand haslpnorm≤ C.lp.tsum_mul_le_mul_norm: basic form of Hölder's inequality
Implementation #
Since lp is defined as an add_subgroup, dot notation does not work. Use lp.norm_neg f to
say that ∥-f∥ = ∥f∥, instead of the non-working f.norm_neg.
TODO #
- More versions of Hölder's inequality (for example: the case
p = 1,q = ∞; a version for normed rings which has∥∑' i, f i * g i∥rather than∑' i, ∥f i∥ * g i∥on the RHS; a version for three exponents satisfying1 / r = 1 / p + 1 / q) - Equivalence with
pi_Lp, forαfinite - Equivalence with
measure_theory.Lp, forf : α → E(i.e., functions rather than pi-types) and the counting measure onα - Equivalence with
bounded_continuous_function, forf : α → E(i.e., functions rather than pi-types) andp = ∞, and the discrete topology onα
The property that f : Π i : α, E i
- is finitely supported, if
p = 0, or - admits an upper bound for
set.range (λ i, ∥f i∥), ifp = ∞, or - has the series
∑' i, ∥f i∥ ^ pbe summable, if0 < p < ∞.
We define pre_lp E to be a type synonym for Π i, E i which, importantly, does not inherit
the pi topology on Π i, E i (otherwise this topology would descend to lp E p and conflict
with the normed group topology we will later equip it with.)
We choose to deal with this issue by making a type synonym for Π i, E i rather than for the lp
subgroup itself, because this allows all the spaces lp E p (for varying p) to be subgroups of
the same ambient group, which permits lemma statements like lp.monotone (below).
Equations
Equations
Equations
- lp.normed_group = normed_group.of_core ↥(lp E p) lp.normed_group._proof_1
Hölder inequality
Equations
- lp.pre_lp.module = pi.module α E 𝕜
The 𝕜-submodule of elements of Π i : α, E i whose lp norm is finite. This is lp E p,
with extra structure.
Equations
- lp.module = {to_distrib_mul_action := module.to_distrib_mul_action (lp.lp_submodule E p 𝕜).module, add_smul := _, zero_smul := _}
Equations
- lp.normed_space = {to_module := lp.module (λ (i : α), _inst_3 i), norm_smul_le := _}
The element of lp E p which is a : E i at the index i, and zero elsewhere.
The canonical finitely-supported approximations to an element f of lp converge to it, in the
lp topology.
The coercion from lp E p to Π i, E i is uniformly continuous.
"Semicontinuity of the lp norm": If all sufficiently large elements of a sequence in lp E p
have lp norm ≤ C, then the pointwise limit, if it exists, also has lp norm ≤ C.
If f is the pointwise limit of a bounded sequence in lp E p, then f is in lp E p.
If a sequence is Cauchy in the lp E p topology and pointwise convergent to a element f of
lp E p, then it converges to f in the lp E p topology.