Documentation

Mathlib.Analysis.SpecialFunctions.Complex.Log

The complex log function #

Basic properties, relationship with exp.

noncomputable def Complex.log (x : ) :

Inverse of the exp function. Returns values such that (log x).im > - π and (log x).im ≤ π. log 0 = 0

Equations
Instances For
    theorem Complex.log_re (x : ) :
    (Complex.log x).re = Real.log (Complex.abs x)
    theorem Complex.exp_log {x : } (hx : x 0) :
    theorem Complex.log_exp {x : } (hx₁ : -Real.pi < x.im) (hx₂ : x.im Real.pi) :
    theorem Complex.exp_inj_of_neg_pi_lt_of_le_pi {x : } {y : } (hx₁ : -Real.pi < x.im) (hx₂ : x.im Real.pi) (hy₁ : -Real.pi < y.im) (hy₂ : y.im Real.pi) (hxy : Complex.exp x = Complex.exp y) :
    x = y
    theorem Complex.ofReal_log {x : } (hx : 0 x) :
    (Real.log x) = Complex.log x
    @[simp]
    theorem Complex.natCast_log {n : } :
    (Real.log n) = Complex.log n
    theorem Complex.log_ofReal_mul {r : } (hr : 0 < r) {x : } (hx : x 0) :
    Complex.log (r * x) = (Real.log r) + Complex.log x
    theorem Complex.log_mul_ofReal (r : ) (hr : 0 < r) (x : ) (hx : x 0) :
    Complex.log (x * r) = (Real.log r) + Complex.log x
    theorem Complex.log_mul {x : } {y : } (hx₀ : x 0) (hy₀ : y 0) :

    Alias of the reverse direction of Complex.log_mul_eq_add_log_iff.

    @[simp]
    @[simp]
    theorem Complex.exp_eq_one_iff {x : } :
    Complex.exp x = 1 ∃ (n : ), x = n * (2 * Real.pi * Complex.I)
    theorem Complex.exp_eq_exp_iff_exists_int {x : } {y : } :
    Complex.exp x = Complex.exp y ∃ (n : ), x = y + n * (2 * Real.pi * Complex.I)
    theorem Complex.tendsto_log_nhdsWithin_im_neg_of_re_neg_of_im_zero {z : } (hre : z.re < 0) (him : z.im = 0) :
    Filter.Tendsto Complex.log (nhdsWithin z {z : | z.im < 0}) (nhds ((Real.log (Complex.abs z)) - Real.pi * Complex.I))
    theorem Complex.continuousWithinAt_log_of_re_neg_of_im_zero {z : } (hre : z.re < 0) (him : z.im = 0) :
    theorem Complex.tendsto_log_nhdsWithin_im_nonneg_of_re_neg_of_im_zero {z : } (hre : z.re < 0) (him : z.im = 0) :
    Filter.Tendsto Complex.log (nhdsWithin z {z : | 0 z.im}) (nhds ((Real.log (Complex.abs z)) + Real.pi * Complex.I))
    theorem Filter.Tendsto.clog {α : Type u_1} {l : Filter α} {f : α} {x : } (h : Filter.Tendsto f l (nhds x)) (hx : x Complex.slitPlane) :
    Filter.Tendsto (fun (t : α) => Complex.log (f t)) l (nhds (Complex.log x))
    theorem ContinuousAt.clog {α : Type u_1} [TopologicalSpace α] {f : α} {x : α} (h₁ : ContinuousAt f x) (h₂ : f x Complex.slitPlane) :
    ContinuousAt (fun (t : α) => Complex.log (f t)) x
    theorem ContinuousWithinAt.clog {α : Type u_1} [TopologicalSpace α] {f : α} {s : Set α} {x : α} (h₁ : ContinuousWithinAt f s x) (h₂ : f x Complex.slitPlane) :
    ContinuousWithinAt (fun (t : α) => Complex.log (f t)) s x
    theorem ContinuousOn.clog {α : Type u_1} [TopologicalSpace α] {f : α} {s : Set α} (h₁ : ContinuousOn f s) (h₂ : xs, f x Complex.slitPlane) :
    ContinuousOn (fun (t : α) => Complex.log (f t)) s
    theorem Continuous.clog {α : Type u_1} [TopologicalSpace α] {f : α} (h₁ : Continuous f) (h₂ : ∀ (x : α), f x Complex.slitPlane) :
    Continuous fun (t : α) => Complex.log (f t)