Extending an ℝ
-linear functional to a 𝕜
-linear functional #
In this file we provide a way to extend a (optionally, continuous) ℝ
-linear map to a (continuous)
𝕜
-linear map in a way that bounds the norm by the norm of the original map, when 𝕜
is either
ℝ
(the extension is trivial) or ℂ
. We formulate the extension uniformly, by assuming RCLike 𝕜
.
We motivate the form of the extension as follows. Note that fc : F →ₗ[𝕜] 𝕜
is determined fully by
re fc
: for all x : F
, fc (I • x) = I * fc x
, so im (fc x) = -re (fc (I • x))
. Therefore,
given an fr : F →ₗ[ℝ] ℝ
, we define fc x = fr x - fr (I • x) * I
.
In Analysis/Normed/Module/RCLike/Extend.lean
we show that this extension is isometric.
This is separate to avoid importing material about the operator norm into files about more
elementary properties, like locally convex spaces.
Main definitions #
Implementation details #
For convenience, the main definitions above operate in terms of RestrictScalars ℝ 𝕜 F
.
Alternate forms which operate on [IsScalarTower ℝ 𝕜 F]
instead are provided with a primed name.
Extend fr : Dual ℝ F
to Dual 𝕜 F
in a way that will also be continuous and have its norm
(as a continuous linear map) equal to ‖fr‖
when fr
is itself continuous on a normed space.
Equations
Instances For
Equations
Extend fr : Dual ℝ (RestrictScalars ℝ 𝕜 F)
to Dual 𝕜 F
.
Equations
Instances For
Extend fr : StrongDual ℝ F
to StrongDual 𝕜 F
.
It would be possible to use LinearMap.mkContinuous
here, but we would need to know that the
continuity of fr
implies it has bounded norm and we want to avoid that dependency here.
Norm properties of this extension can be found in
Mathlib/Analysis/Normed/Module/RCLike/Extend.lean
.
Equations
- ContinuousLinearMap.extendTo𝕜' fr = { toLinearMap := (↑fr).extendTo𝕜', cont := ⋯ }
Instances For
Extend fr : StrongDual ℝ (RestrictScalars ℝ 𝕜 F)
to StrongDual 𝕜 F
.