Documentation

Mathlib.Analysis.SpecialFunctions.Complex.Circle

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 (-π, π].

@[simp]
theorem Circle.arg_eq_arg {z w : Circle} :
(↑z).arg = (↑w).arg z = w
theorem Circle.arg_exp {x : } (h₁ : -Real.pi < x) (h₂ : x Real.pi) :
(↑(exp x)).arg = x
@[simp]
theorem Circle.exp_arg (z : Circle) :
exp (↑z).arg = z

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
    noncomputable def Circle.argEquiv :

    Complex.arg and expMapCircle define an equivalence between circle and (-π, π].

    Equations
    Instances For
      @[simp]
      theorem Circle.argEquiv_apply_coe (z : Circle) :
      (argEquiv z) = (↑z).arg
      theorem Circle.exp_eq_exp {x y : } :
      exp x = exp y ∃ (m : ), x = y + m * (2 * Real.pi)
      @[simp]
      theorem Circle.exp_int_mul_two_pi (n : ) :
      exp (n * (2 * Real.pi)) = 1
      theorem Circle.exp_two_pi_mul_int (n : ) :
      exp (2 * Real.pi * n) = 1
      theorem Circle.exp_eq_one {r : } :
      exp r = 1 ∃ (n : ), r = n * (2 * Real.pi)
      theorem Circle.exp_inj {r s : } :
      noncomputable def Real.Angle.toCircle (θ : Angle) :

      Circle.exp, applied to a Real.Angle.

      Equations
      Instances For
        @[simp]
        theorem Real.Angle.coe_toCircle (θ : Angle) :
        θ.toCircle = θ.cos + θ.sin * Complex.I
        @[simp]
        theorem Real.Angle.toCircle_add (θ₁ θ₂ : Angle) :
        (θ₁ + θ₂).toCircle = θ₁.toCircle * θ₂.toCircle
        @[simp]
        theorem Real.Angle.arg_toCircle (θ : Angle) :
        (↑θ.toCircle).arg = θ

        Map from AddCircle to Circle #

        noncomputable def AddCircle.toCircle {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]

          The homeomorphism between AddCircle (2 * π) and Circle.

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