Maps on the unit circle #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we prove some basic lemmas about exp_map_circle
and the restriction of complex.arg
to the unit circle. These two maps define a local equivalence between circle
and ℝ
, see
circle.arg_local_equiv
and circle.arg_equiv
, that sends the whole circle to (-π, π]
.
@[simp]
complex.arg ∘ coe
and exp_map_circle
define a local equivalence between circle and
ℝwith
source = set.univand
target = set.Ioc (-π) π`.
Equations
- circle.arg_local_equiv = {to_fun := complex.arg ∘ coe, inv_fun := ⇑exp_map_circle, source := set.univ ↥circle, target := set.Ioc (-real.pi) real.pi, map_source' := circle.arg_local_equiv._proof_1, map_target' := circle.arg_local_equiv._proof_2, left_inv' := circle.arg_local_equiv._proof_3, right_inv' := circle.arg_local_equiv._proof_4}
@[simp]
@[simp]
complex.arg
and exp_map_circle
define an equivalence between circle and
(-π, π]`.
exp_map_circle
, applied to a real.angle
.
Equations
@[simp]
@[simp]
@[simp]
theorem
real.angle.exp_map_circle_add
(θ₁ θ₂ : real.angle) :
(θ₁ + θ₂).exp_map_circle = θ₁.exp_map_circle * θ₂.exp_map_circle
@[simp]