Mazur-Ulam Theorem #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
Mazur-Ulam theorem states that an isometric bijection between two normed affine spaces over ℝ
is
affine. We formalize it in three definitions:
isometry_equiv.to_real_linear_isometry_equiv_of_map_zero
: givenE ≃ᵢ F
sending0
to0
, returnsE ≃ₗᵢ[ℝ] F
with the sameto_fun
andinv_fun
;isometry_equiv.to_real_linear_isometry_equiv
: givenf : E ≃ᵢ F
, returns a linear isometry equivalenceg : E ≃ₗᵢ[ℝ] F
withg x = f x - f 0
.isometry_equiv.to_real_affine_isometry_equiv
: givenf : PE ≃ᵢ PF
, returns an affine isometry equivalenceg : PE ≃ᵃⁱ[ℝ] PF
whose underlyingisometry_equiv
isf
The formalization is based on Jussi Väisälä, A Proof of the Mazur-Ulam Theorem.
Tags #
isometry, affine map, linear map
If an isometric self-homeomorphism of a normed vector space over ℝ
fixes x
and y
,
then it fixes the midpoint of [x, y]
. This is a lemma for a more general Mazur-Ulam theorem,
see below.
A bijective isometry sends midpoints to midpoints.
Since f : PE ≃ᵢ PF
sends midpoints to midpoints, it is an affine map.
We define a conversion to a continuous_linear_equiv
first, then a conversion to an affine_map
.
Mazur-Ulam Theorem: if f
is an isometric bijection between two normed vector spaces
over ℝ
and f 0 = 0
, then f
is a linear isometry equivalence.
Equations
- f.to_real_linear_isometry_equiv_of_map_zero h0 = {to_linear_equiv := {to_fun := ((add_monoid_hom.of_map_midpoint ℝ ℝ ⇑f h0 _).to_real_linear_map _).to_linear_map.to_fun, map_add' := _, map_smul' := _, inv_fun := f.to_equiv.inv_fun, left_inv := _, right_inv := _}, norm_map' := _}
Mazur-Ulam Theorem: if f
is an isometric bijection between two normed vector spaces
over ℝ
, then x ↦ f x - f 0
is a linear isometry equivalence.
Equations
Mazur-Ulam Theorem: if f
is an isometric bijection between two normed add-torsors over
normed vector spaces over ℝ
, then f
is an affine isometry equivalence.