Documentation

Mathlib.Analysis.SpecialFunctions.Complex.Arg

The argument of a complex number. #

We define arg : ℂ → ℝ, returning a real number in the range (-π, π], such that for x ≠ 0, sin (arg x) = x.im / x.abs and cos (arg x) = x.re / x.abs, while arg 0 defaults to 0

noncomputable def Complex.arg (x : ) :

arg returns values in the range (-π, π], such that for x ≠ 0, sin (arg x) = x.im / x.abs and cos (arg x) = x.re / x.abs, arg 0 defaults to 0

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem Complex.sin_arg (x : ) :
    Real.sin (Complex.arg x) = x.im / Complex.abs x
    theorem Complex.cos_arg {x : } (hx : x 0) :
    Real.cos (Complex.arg x) = x.re / Complex.abs x
    @[simp]
    theorem Complex.abs_mul_exp_arg_mul_I (x : ) :
    (Complex.abs x) * Complex.exp ((Complex.arg x) * Complex.I) = x
    @[simp]
    theorem Complex.abs_mul_cos_add_sin_mul_I (x : ) :
    (Complex.abs x) * (Complex.cos (Complex.arg x) + Complex.sin (Complex.arg x) * Complex.I) = x
    @[simp]
    theorem Complex.abs_mul_cos_arg (x : ) :
    Complex.abs x * Real.cos (Complex.arg x) = x.re
    @[simp]
    theorem Complex.abs_mul_sin_arg (x : ) :
    Complex.abs x * Real.sin (Complex.arg x) = x.im
    theorem Complex.abs_eq_one_iff (z : ) :
    Complex.abs z = 1 ∃ (θ : ), Complex.exp (θ * Complex.I) = z
    theorem Complex.arg_mul_cos_add_sin_mul_I {r : } (hr : 0 < r) {θ : } (hθ : θ Set.Ioc (-Real.pi) Real.pi) :
    Complex.arg (r * (Complex.cos θ + Complex.sin θ * Complex.I)) = θ
    @[simp]
    theorem Complex.ext_abs_arg {x : } {y : } (h₁ : Complex.abs x = Complex.abs y) (h₂ : Complex.arg x = Complex.arg y) :
    x = y
    theorem Complex.ext_abs_arg_iff {x : } {y : } :
    x = y Complex.abs x = Complex.abs y Complex.arg x = Complex.arg y
    @[simp]
    theorem Complex.arg_nonneg_iff {z : } :
    0 Complex.arg z 0 z.im
    @[simp]
    theorem Complex.arg_neg_iff {z : } :
    Complex.arg z < 0 z.im < 0
    theorem Complex.arg_real_mul (x : ) {r : } (hr : 0 < r) :
    theorem Complex.arg_mul_real {r : } (hr : 0 < r) (x : ) :
    theorem Complex.arg_eq_arg_iff {x : } {y : } (hx : x 0) (hy : y 0) :
    Complex.arg x = Complex.arg y (Complex.abs y) / (Complex.abs x) * x = y
    @[simp]
    @[simp]
    theorem Complex.tan_arg (x : ) :
    Real.tan (Complex.arg x) = x.im / x.re
    theorem Complex.arg_ofReal_of_nonneg {x : } (hx : 0 x) :
    Complex.arg x = 0
    @[simp]
    theorem Complex.natCast_arg {n : } :
    Complex.arg n = 0
    theorem Complex.arg_eq_zero_iff {z : } :
    Complex.arg z = 0 0 z.re z.im = 0
    theorem Complex.arg_eq_pi_iff {z : } :
    Complex.arg z = Real.pi z.re < 0 z.im = 0
    theorem Complex.arg_ofReal_of_neg {x : } (hx : x < 0) :
    theorem Complex.arg_of_re_nonneg {x : } (hx : 0 x.re) :
    Complex.arg x = Real.arcsin (x.im / Complex.abs x)
    theorem Complex.arg_of_re_neg_of_im_nonneg {x : } (hx_re : x.re < 0) (hx_im : 0 x.im) :
    Complex.arg x = Real.arcsin ((-x).im / Complex.abs x) + Real.pi
    theorem Complex.arg_of_re_neg_of_im_neg {x : } (hx_re : x.re < 0) (hx_im : x.im < 0) :
    Complex.arg x = Real.arcsin ((-x).im / Complex.abs x) - Real.pi
    theorem Complex.arg_of_im_nonneg_of_ne_zero {z : } (h₁ : 0 z.im) (h₂ : z 0) :
    Complex.arg z = Real.arccos (z.re / Complex.abs z)
    theorem Complex.arg_of_im_pos {z : } (hz : 0 < z.im) :
    Complex.arg z = Real.arccos (z.re / Complex.abs z)
    theorem Complex.arg_of_im_neg {z : } (hz : z.im < 0) :
    Complex.arg z = -Real.arccos (z.re / Complex.abs z)
    theorem Complex.abs_eq_one_iff' {x : } :
    Complex.abs x = 1 ∃ θ ∈ Set.Ioc (-Real.pi) Real.pi, Complex.exp (θ * Complex.I) = x
    theorem Complex.arg_lt_pi_div_two_iff {z : } :
    Complex.arg z < Real.pi / 2 0 < z.re z.im < 0 z = 0
    @[simp]
    theorem Complex.arg_neg_coe_angle {x : } (hx : x 0) :
    (Complex.arg (-x)) = (Complex.arg x) + Real.pi
    theorem Complex.arg_mul_cos_add_sin_mul_I_sub {r : } (hr : 0 < r) (θ : ) :
    Complex.arg (r * (Complex.cos θ + Complex.sin θ * Complex.I)) - θ = 2 * Real.pi * (Real.pi - θ) / (2 * Real.pi)
    theorem Complex.arg_mul_cos_add_sin_mul_I_coe_angle {r : } (hr : 0 < r) (θ : Real.Angle) :
    (Complex.arg (r * ((Real.Angle.cos θ) + (Real.Angle.sin θ) * Complex.I))) = θ
    theorem Complex.arg_mul_coe_angle {x : } {y : } (hx : x 0) (hy : y 0) :
    (Complex.arg (x * y)) = (Complex.arg x) + (Complex.arg y)
    theorem Complex.arg_div_coe_angle {x : } {y : } (hx : x 0) (hy : y 0) :
    (Complex.arg (x / y)) = (Complex.arg x) - (Complex.arg y)
    theorem Complex.arg_mul {x : } {y : } (hx₀ : x 0) (hy₀ : y 0) :

    Alias of the reverse direction of Complex.arg_mul_eq_add_arg_iff.

    An alternative description of the slit plane as consisting of nonzero complex numbers whose argument is not π.

    theorem Complex.arg_eq_nhds_of_re_pos {x : } (hx : 0 < x.re) :
    Complex.arg =ᶠ[nhds x] fun (x : ) => Real.arcsin (x.im / Complex.abs x)
    theorem Complex.arg_eq_nhds_of_re_neg_of_im_pos {x : } (hx_re : x.re < 0) (hx_im : 0 < x.im) :
    Complex.arg =ᶠ[nhds x] fun (x : ) => Real.arcsin ((-x).im / Complex.abs x) + Real.pi
    theorem Complex.arg_eq_nhds_of_re_neg_of_im_neg {x : } (hx_re : x.re < 0) (hx_im : x.im < 0) :
    Complex.arg =ᶠ[nhds x] fun (x : ) => Real.arcsin ((-x).im / Complex.abs x) - Real.pi
    theorem Complex.arg_eq_nhds_of_im_pos {z : } (hz : 0 < z.im) :
    Complex.arg =ᶠ[nhds z] fun (x : ) => Real.arccos (x.re / Complex.abs x)
    theorem Complex.arg_eq_nhds_of_im_neg {z : } (hz : z.im < 0) :
    Complex.arg =ᶠ[nhds z] fun (x : ) => -Real.arccos (x.re / Complex.abs x)
    theorem Complex.continuousWithinAt_arg_of_re_neg_of_im_zero {z : } (hre : z.re < 0) (him : z.im = 0) :