Operator norm on the space of continuous linear maps #
Define the operator (semi)-norm on the space of continuous (semi)linear maps between (semi)-normed spaces, and prove its basic properties. In particular, show that this space is itself a semi-normed space.
Since a lot of elementary properties don't require βxβ = 0 β x = 0 we start setting up the
theory for SeminormedAddCommGroup. Later we will specialize to NormedAddCommGroup in the
file NormedSpace.lean.
Note that most of statements that apply to semilinear maps only hold when the ring homomorphism
is isometric, as expressed by the typeclass [RingHomIsometric Ο].
If βxβ = 0 and f is continuous then βf xβ = 0.
A continuous linear map between seminormed spaces is bounded when the field is nontrivially
normed. The continuity ensures boundedness on a ball of some radius Ξ΅. The nontriviality of the
norm 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.
Given a unit-length element x of a normed space E over a field π, the natural linear
isometry map from π to E by taking multiples of x.
Equations
- LinearIsometry.toSpanSingleton π E hv = let __src := LinearMap.toSpanSingleton π E v; { toLinearMap := __src, norm_map' := β― }
Instances For
The operator norm of a continuous linear map is the inf of all its bounds.
Instances For
Equations
- ContinuousLinearMap.hasOpNorm = { norm := ContinuousLinearMap.opNorm }
Alias of ContinuousLinearMap.isLeast_opNorm.
If one controls the norm of every A x, then one controls the norm of A.
Alias of ContinuousLinearMap.opNorm_le_bound.
If one controls the norm of every A x, then one controls the norm of A.
If one controls the norm of every A x, βxβ β  0, then one controls the norm of A.
Alias of ContinuousLinearMap.opNorm_le_bound'.
If one controls the norm of every A x, βxβ β  0, then one controls the norm of A.
Alias of ContinuousLinearMap.opNorm_eq_of_bounds.
Alias of ContinuousLinearMap.opNorm_neg.
Alias of ContinuousLinearMap.opNorm_nonneg.
The norm of the 0 operator is 0.
Alias of ContinuousLinearMap.opNorm_zero.
The norm of the 0 operator is 0.
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.
The fundamental property of the operator norm: βf xβ β€ βfβ * βxβ.
Alias of ContinuousLinearMap.le_opNorm.
The fundamental property of the operator norm: βf xβ β€ βfβ * βxβ.
Alias of ContinuousLinearMap.dist_le_opNorm.
Alias of ContinuousLinearMap.le_opNorm_of_le.
Alias of ContinuousLinearMap.le_of_opNorm_le.
Alias of ContinuousLinearMap.opNorm_le_iff.
Alias of ContinuousLinearMap.ratio_le_opNorm.
The image of the unit ball under a continuous linear map is bounded.
Alias of ContinuousLinearMap.unit_le_opNorm.
The image of the unit ball under a continuous linear map is bounded.
Alias of ContinuousLinearMap.opNorm_le_of_shell.
Alias of ContinuousLinearMap.opNorm_le_of_ball.
Alias of ContinuousLinearMap.opNorm_le_of_shell'.
For a continuous real linear map f, if one controls the norm of every f x, βxβ = 1, then
one controls the norm of f.
Alias of ContinuousLinearMap.opNorm_le_of_unit_norm.
For a continuous real linear map f, if one controls the norm of every f x, βxβ = 1, then
one controls the norm of f.
The operator norm satisfies the triangle inequality.
Alias of ContinuousLinearMap.opNorm_add_le.
The operator norm satisfies the triangle inequality.
If there is an element with norm different from 0, then the norm of the identity equals 1.
(Since we are working with seminorms supposing that the space is non-trivial is not enough.)
Alias of ContinuousLinearMap.opNorm_smul_le.
Operator seminorm on the space of continuous (semi)linear maps, as Seminorm.
We use this seminorm to define a SeminormedGroup structure on E βSL[Ο] F,
but we have to override the projection UniformSpace
so that it is definitionally equal to the one coming from the topologies on E and F.
Equations
- ContinuousLinearMap.seminorm = Seminorm.ofSMulLE norm β― β― β―
Instances For
Equations
- ContinuousLinearMap.toPseudoMetricSpace = SeminormedAddCommGroup.toPseudoMetricSpace.replaceUniformity β―
Continuous linear maps themselves form a seminormed space with respect to the operator norm.
Equations
- ContinuousLinearMap.toSeminormedAddCommGroup = SeminormedAddCommGroup.mk β―
Equations
- ContinuousLinearMap.toNormedSpace = NormedSpace.mk β―
The operator norm is submultiplicative.
Alias of ContinuousLinearMap.opNorm_comp_le.
The operator norm is submultiplicative.
Continuous linear maps form a seminormed ring with respect to the operator norm.
Equations
- ContinuousLinearMap.toSemiNormedRing = let __src := ContinuousLinearMap.toSeminormedAddCommGroup; let __src_1 := ContinuousLinearMap.ring; SeminormedRing.mk β― β―
For a normed space E, continuous linear endomorphisms form a normed algebra with
respect to the operator norm.
Equations
- ContinuousLinearMap.toNormedAlgebra = let __src := ContinuousLinearMap.algebra; NormedAlgebra.mk β―
Alias of ContinuousLinearMap.opNorm_subsingleton.
ContinuousLinearMap.restrictScalars as a LinearIsometry.
Equations
- ContinuousLinearMap.restrictScalarsIsometry π E Fβ π' π'' = { toLinearMap := ContinuousLinearMap.restrictScalarsβ π E Fβ π' π'', norm_map' := β― }
Instances For
ContinuousLinearMap.restrictScalars as a ContinuousLinearMap.
Equations
- ContinuousLinearMap.restrictScalarsL π E Fβ π' π'' = (ContinuousLinearMap.restrictScalarsIsometry π E Fβ π' π'').toContinuousLinearMap
Instances For
If a continuous linear map is constructed from a linear map via the constructor mkContinuous,
then its norm is bounded by the bound given to the constructor if it is nonnegative.
If a continuous linear map is constructed from a linear map via the constructor mkContinuous,
then its norm is bounded by the bound or zero if bound is negative.