Operator norm on the space of continuous linear maps
Define the operator norm on the space of continuous linear maps between normed spaces, and prove its basic properties. In particular, show that this space is itself a normed space.
Construct a continuous linear map from a linear map and a bound on this linear map.
The fact that the norm of the continuous linear map is then controlled is given in
linear_map.mk_continuous_norm_le
.
Equations
- f.mk_continuous C h = {to_linear_map := f, cont := _}
Reinterpret a linear map 𝕜 →ₗ[𝕜] E
as a continuous linear map. This construction
is generalized to the case of any finite dimensional domain
in linear_map.to_continuous_linear_map
.
Equations
- f.to_continuous_linear_map₁ = f.mk_continuous ∥⇑f 1∥ _
Construct a continuous linear map from a linear map and the existence of a bound on this linear
map. If you have an explicit bound, use linear_map.mk_continuous
instead, as a norm estimate will
follow automatically in linear_map.mk_continuous_norm_le
.
Equations
- f.mk_continuous_of_exists_bound h = {to_linear_map := f, cont := _}
- _ = _
A continuous linear map between normed spaces is bounded when the field is nondiscrete.
The continuity ensures boundedness on a ball of some radius δ
. The nondiscreteness is then
used to rescale any element into an element of norm in [δ/C, δ]
, whose image has a controlled norm.
The norm control for the original element follows by rescaling.
A linear map which is a homothety is a continuous linear map.
Since the field 𝕜
need not have ℝ
as a subfield, this theorem is not directly deducible from
the corresponding theorem about isometries plus a theorem about scalar multiplication. Likewise
for the other theorems about homotheties in this file.
Equations
- continuous_linear_map.of_homothety f a hf = f.mk_continuous a _
Given an element x
of a normed space E
over a field 𝕜
, the natural continuous
linear map from E
to the span of x
.
Equations
The operator norm of a continuous linear map is the inf of all its bounds.
Equations
The fundamental property of the operator norm: ∥f x∥ ≤ ∥f∥ * ∥x∥
.
continuous linear maps are Lipschitz continuous.
The image of the unit ball under a continuous linear map is bounded.
If one controls the norm of every A x
, then one controls the norm of A
.
The operator norm satisfies the triangle inequality.
An operator is zero iff its norm vanishes.
The norm of the identity is at most 1
. It is in fact 1
, except when the space is trivial
where it is 0
. It means that one can not do better than an inequality in general.
If a space is non-trivial, then the norm of the identity equals 1
.
Continuous linear maps themselves form a normed space with respect to the operator norm.
Equations
- continuous_linear_map.to_normed_group = normed_group.of_core (E →L[𝕜] F) continuous_linear_map.to_normed_group._proof_1
The operator norm is submultiplicative.
Continuous linear maps form a normed ring with respect to the operator norm.
Equations
For a nonzero normed space E
, continuous linear endomorphisms form a normed algebra with
respect to the operator norm.
A continuous linear map is automatically uniformly continuous.
A continuous linear map is an isometry if and only if it preserves the norm.
If a continuous linear map is a uniform embedding, then it is expands the distances by a positive factor.
If the target space is complete, the space of continuous linear maps with its norm is also complete.
Equations
Extension of a continuous linear map f : E →L[𝕜] F
, with E
a normed space and F
a complete
normed space, along a uniform and dense embedding e : E →L[𝕜] G
.
If a dense embedding e : E →L[𝕜] G
expands the norm by a constant factor N⁻¹
, then the norm
of the extension of f
along e
is bounded by N * ∥f∥
.
If a continuous linear map is constructed from a linear map via the constructor mk_continuous
,
then its norm is bounded by the bound given to the constructor if it is nonnegative.
The norm of the tensor product of a scalar linear map and of an element of a normed space is the product of the norms.
Left-multiplication in a normed algebra, considered as a continuous linear map.
Equations
- continuous_linear_map.lmul_left 𝕜 𝕜' = λ (x : 𝕜'), (algebra.lmul_left 𝕜 𝕜' x).mk_continuous ∥x∥ _
Right-multiplication in a normed algebra, considered as a continuous linear map.
Equations
- continuous_linear_map.lmul_right 𝕜 𝕜' = λ (x : 𝕜'), (algebra.lmul_right 𝕜 𝕜' x).mk_continuous ∥x∥ _
Simultaneous left- and right-multiplication in a normed algebra, considered as a continuous linear map.
Equations
- continuous_linear_map.lmul_left_right 𝕜 𝕜' vw = (continuous_linear_map.lmul_right 𝕜 𝕜' vw.snd).comp (continuous_linear_map.lmul_left 𝕜 𝕜' vw.fst)
𝕜
-linear continuous function induced by a 𝕜'
-linear continuous function when 𝕜'
is a
normed algebra over 𝕜
.
Equations
- continuous_linear_map.restrict_scalars 𝕜 f = {to_linear_map := {to_fun := (linear_map.restrict_scalars 𝕜 f.to_linear_map).to_fun, map_add' := _, map_smul' := _}, cont := _}
Equations
- continuous_linear_map.has_scalar_extend_scalars = {smul := λ (c : 𝕜') (f : E →L[𝕜] semimodule.restrict_scalars 𝕜 𝕜' F'), (c • f.to_linear_map).mk_continuous (∥c∥ * ∥f∥) _}
Equations
- continuous_linear_map.module_extend_scalars = {to_distrib_mul_action := {to_mul_action := {to_has_scalar := continuous_linear_map.has_scalar_extend_scalars _inst_11, one_smul := _, mul_smul := _}, smul_add := _, smul_zero := _}, add_smul := _, zero_smul := _}
Equations
When f
is a continuous linear map taking values in S
, then λb, f b • x
is a
continuous linear map.
Equations
- f.smul_algebra_right x = {to_linear_map := {to_fun := (smul_algebra_right f.to_linear_map x).to_fun, map_add' := _, map_smul' := _}, cont := _}
Applying a continuous linear map commutes with taking an (infinite) sum.
A continuous linear equiv is a uniform embedding.
A linear equivalence which is a homothety is a continuous linear equivalence.
Equations
- continuous_linear_equiv.of_homothety 𝕜 f a ha hf = {to_linear_equiv := f, continuous_to_fun := _, continuous_inv_fun := _}
Given a nonzero element x
of a normed space E
over a field 𝕜
, the natural
continuous linear equivalence from E
to the span of x
.
Equations
Given a nonzero element x
of a normed space E
over a field 𝕜
, the natural continuous
linear map from the span of x
to 𝕜
.
The continuous linear equivalences from E
to itself form a group under composition.
Equations
- continuous_linear_equiv.automorphism_group 𝕜 E = {mul := λ (f g : E ≃L[𝕜] E), g.trans f, mul_assoc := _, one := continuous_linear_equiv.refl 𝕜 E normed_space.to_semimodule, one_mul := _, mul_one := _, inv := λ (f : E ≃L[𝕜] E), f.symm, mul_left_inv := _}
An invertible continuous linear map f
determines a continuous equivalence from E
to itself.
Equations
- continuous_linear_equiv.of_unit f = {to_linear_equiv := {to_fun := ⇑(f.val), map_add' := _, map_smul' := _, inv_fun := ⇑(f.inv), left_inv := _, right_inv := _}, continuous_to_fun := _, continuous_inv_fun := _}
A continuous equivalence from E
to itself determines an invertible continuous linear map.
The units of the algebra of continuous 𝕜
-linear endomorphisms of E
is multiplicatively
equivalent to the type of continuous linear equivalences between E
and itself.
Equations
- continuous_linear_equiv.units_equiv 𝕜 E = {to_fun := continuous_linear_equiv.of_unit _inst_5, inv_fun := continuous_linear_equiv.to_unit _inst_5, left_inv := _, right_inv := _, map_mul' := _}