Documentation

Mathlib.Analysis.NormedSpace.MazurUlam

Mazur-Ulam Theorem #

Mazur-Ulam theorem states that an isometric bijection between two normed affine spaces over is affine. We formalize it in three definitions:

The formalization is based on [Jussi Väisälä, A Proof of the Mazur-Ulam Theorem][Vaisala_2003].

Tags #

isometry, affine map, linear map

theorem IsometryEquiv.midpoint_fixed {E : Type u_1} {PE : Type u_2} [NormedAddCommGroup E] [NormedSpace E] [MetricSpace PE] [NormedAddTorsor E PE] {x : PE} {y : PE} (e : PE ≃ᵢ PE) :
e x = xe y = ye (midpoint x y) = midpoint x y

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.

theorem IsometryEquiv.map_midpoint {E : Type u_1} {PE : Type u_2} {F : Type u_3} {PF : Type u_4} [NormedAddCommGroup E] [NormedSpace E] [MetricSpace PE] [NormedAddTorsor E PE] [NormedAddCommGroup F] [NormedSpace F] [MetricSpace PF] [NormedAddTorsor F PF] (f : PE ≃ᵢ PF) (x : PE) (y : PE) :
f (midpoint x y) = midpoint (f x) (f y)

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 ContinuousLinearEquiv first, then a conversion to an AffineMap.

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
  • One or more equations did not get rendered due to their size.
Instances For

    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
    Instances For

      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.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For