Maps on the unit circle #
In this file we prove some basic lemmas about expMapCircle
and the restriction of Complex.arg
to the unit circle. These two maps define a partial equivalence between circle
and ℝ
, see
circle.argPartialEquiv
and circle.argEquiv
, that sends the whole circle to (-π, π]
.
Complex.arg ∘ (↑)
and expMapCircle
define a partial equivalence between circle
and ℝ
with source = Set.univ
and target = Set.Ioc (-π) π
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
Complex.arg
and expMapCircle
define an equivalence between circle
and (-π, π]
.
Equations
- Circle.argEquiv = { toFun := fun (z : Circle) => ⟨(↑z).arg, ⋯⟩, invFun := ⇑Circle.exp ∘ Subtype.val, left_inv := ⋯, right_inv := Circle.argEquiv.proof_2 }
Instances For
theorem
Circle.invOn_arg_exp :
Set.InvOn (Complex.arg ∘ Subtype.val) (⇑exp) (Set.Ioc (-Real.pi) Real.pi) Set.univ
theorem
AddCircle.scaled_exp_map_periodic
{T : ℝ}
:
Function.Periodic (fun (x : ℝ) => Circle.exp (2 * Real.pi / T * x)) T
The canonical map fun x => exp (2 π i x / T)
from ℝ / ℤ • T
to the unit circle in ℂ
.
If T = 0
we understand this as the constant function 1.
Equations
Instances For
@[simp]
@[simp]