Isometries of the Complex Plane #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
The lemma linear_isometry_complex
states the classification of isometries in the complex plane.
Specifically, isometries with rotations but without translation.
The proof involves:
- creating a linear isometry
g
with two fixed points,g(0) = 0
,g(1) = 1
- applying
linear_isometry_complex_aux
tog
The proof oflinear_isometry_complex_aux
is separated in the following parts: - show that the real parts match up:
linear_isometry.re_apply_eq_re
- show that I maps to either I or -I
- every z is a linear combination of a + b * I
References #
An element of the unit circle defines a linear_isometry_equiv
from ℂ
to itself, by
rotation.
Equations
- rotation = {to_fun := λ (a : ↥circle), {to_linear_equiv := {to_fun := (distrib_mul_action.to_linear_equiv ℝ ℂ a).to_fun, map_add' := _, map_smul' := _, inv_fun := (distrib_mul_action.to_linear_equiv ℝ ℂ a).inv_fun, left_inv := _, right_inv := _}, norm_map' := _}, map_one' := rotation._proof_7, map_mul' := rotation._proof_8}
The matrix representation of rotation a
is equal to the conformal matrix
!![re a, -im a; im a, re a]
.
@[simp]
The determinant of rotation
(as a linear map) is equal to 1
.
@[simp]
The determinant of rotation
(as a linear equiv) is equal to 1
.