Continuous affine maps between normed spaces. #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file develops the theory of continuous affine maps between affine spaces modelled on normed spaces.
In the particular case that the affine spaces are just normed vector spaces V
, W
, we define a
norm on the space of continuous affine maps by defining the norm of f : V →A[𝕜] W
to be
‖f‖ = max ‖f 0‖ ‖f.cont_linear‖
. This is chosen so that we have a linear isometry:
(V →A[𝕜] W) ≃ₗᵢ[𝕜] W × (V →L[𝕜] W)
.
The abstract picture is that for an affine space P
modelled on a vector space V
, together with
a vector space W
, there is an exact sequence of 𝕜
-modules: 0 → C → A → L → 0
where C
, A
are the spaces of constant and affine maps P → W
and L
is the space of linear maps V → W
.
Any choice of a base point in P
corresponds to a splitting of this sequence so in particular if we
take P = V
, using 0 : V
as the base point provides a splitting, and we prove this is an
isometric decomposition.
On the other hand, choosing a base point breaks the affine invariance so the norm fails to be
submultiplicative: for a composition of maps, we have only ‖f.comp g‖ ≤ ‖f‖ * ‖g‖ + ‖f 0‖
.
Main definitions: #
The linear map underlying a continuous affine map is continuous.
Equations
- f.cont_linear = {to_linear_map := {to_fun := ⇑(f.to_affine_map.linear), map_add' := _, map_smul' := _}, cont := _}
Note that unlike the operator norm for linear maps, this norm is not submultiplicative:
we do not necessarily have ‖f.comp g‖ ≤ ‖f‖ * ‖g‖
. See norm_comp_le
for what we can say.
Equations
- continuous_affine_map.has_norm = {norm := λ (f : V →A[𝕜] W), linear_order.max ‖⇑f 0‖ ‖f.cont_linear‖}
Equations
- continuous_affine_map.normed_add_comm_group = {to_fun := λ (f : V →A[𝕜] W), linear_order.max ‖⇑f 0‖ ‖f.cont_linear‖, map_zero' := _, add_le' := _, neg' := _, eq_zero_of_map_eq_zero' := _}.to_normed_add_comm_group
Equations
- continuous_affine_map.normed_space = {to_module := continuous_affine_map.module continuous_affine_map.normed_space._proof_3, norm_smul_le := _}
The space of affine maps between two normed spaces is linearly isometric to the product of the
codomain with the space of linear maps, by taking the value of the affine map at (0 : V)
and the
linear part.
Equations
- continuous_affine_map.to_const_prod_continuous_linear_map 𝕜 V W = {to_linear_equiv := {to_fun := λ (f : V →A[𝕜] W), (⇑f 0, f.cont_linear), map_add' := _, map_smul' := _, inv_fun := λ (p : W × (V →L[𝕜] W)), p.snd.to_continuous_affine_map + continuous_affine_map.const 𝕜 V p.fst, left_inv := _, right_inv := _}, norm_map' := _}