The upper half plane and its automorphisms #
This file defines upper_half_plane
to be the upper half plane in ℂ
.
We furthermore equip it with the structure of an SL(2,ℝ)
action by
fractional linear transformations.
We define the notation ℍ
for the upper half plane available in the locale
upper_half_plane
so as not to conflict with the quaternions.
theorem
upper_half_plane.norm_sq_denom_pos
(g : SL(2,ℝ))
(z : ℍ) :
0 < ⇑complex.norm_sq (upper_half_plane.denom g z)
theorem
upper_half_plane.norm_sq_denom_ne_zero
(g : SL(2,ℝ))
(z : ℍ) :
⇑complex.norm_sq (upper_half_plane.denom g z) ≠ 0
Fractional linear transformation
Equations
theorem
upper_half_plane.smul_aux'_im
(g : SL(2,ℝ))
(z : ℍ) :
(upper_half_plane.smul_aux' g z).im = z.im / ⇑complex.norm_sq (upper_half_plane.denom g z)
Fractional linear transformation
Equations
- upper_half_plane.smul_aux g z = ⟨upper_half_plane.smul_aux' g z, _⟩
theorem
upper_half_plane.denom_cocycle
(x y : SL(2,ℝ))
(z : ℍ) :
upper_half_plane.denom (x * y) z = (upper_half_plane.denom x (upper_half_plane.smul_aux y z)) * upper_half_plane.denom y z
theorem
upper_half_plane.mul_smul'
(x y : SL(2,ℝ))
(z : ℍ) :
upper_half_plane.smul_aux (x * y) z = upper_half_plane.smul_aux x (upper_half_plane.smul_aux y z)
@[protected, instance]
The action of SL(2, ℝ)
on the upper half-plane by fractional linear transformations.
Equations
- upper_half_plane.mul_action = {to_has_scalar := {smul := upper_half_plane.smul_aux}, one_smul := upper_half_plane.mul_action._proof_1, mul_smul := upper_half_plane.mul_smul'}
@[simp]
theorem
upper_half_plane.coe_smul
(g : SL(2,ℝ))
(z : ℍ) :
↑(g • z) = upper_half_plane.num g z / upper_half_plane.denom g z
@[simp]
theorem
upper_half_plane.re_smul
(g : SL(2,ℝ))
(z : ℍ) :
(g • z).re = (upper_half_plane.num g z / upper_half_plane.denom g z).re
theorem
upper_half_plane.im_smul
(g : SL(2,ℝ))
(z : ℍ) :
(g • z).im = (upper_half_plane.num g z / upper_half_plane.denom g z).im
theorem
upper_half_plane.im_smul_eq_div_norm_sq
(g : SL(2,ℝ))
(z : ℍ) :
(g • z).im = z.im / ⇑complex.norm_sq (upper_half_plane.denom g z)