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.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
    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
    @[simp]
    @[simp]
    theorem Complex.exp_eq_one_iff {x : } :
    Complex.exp x = 1 n, x = n * (2 * Real.pi * Complex.I)
    theorem Complex.continuousWithinAt_log_of_re_neg_of_im_zero {z : } (hre : z.re < 0) (him : z.im = 0) :
    theorem continuousAt_clog {x : } (h : 0 < x.re x.im 0) :
    theorem Filter.Tendsto.clog {α : Type u_1} {l : Filter α} {f : α} {x : } (h : Filter.Tendsto f l (nhds x)) (hx : 0 < x.re x.im 0) :
    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₂ : 0 < (f x).re (f x).im 0) :
    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₂ : 0 < (f x).re (f x).im 0) :
    ContinuousWithinAt (fun t => Complex.log (f t)) s x
    theorem ContinuousOn.clog {α : Type u_1} [TopologicalSpace α] {f : α} {s : Set α} (h₁ : ContinuousOn f s) (h₂ : ∀ (x : α), x s0 < (f x).re (f x).im 0) :
    ContinuousOn (fun t => Complex.log (f t)) s
    theorem Continuous.clog {α : Type u_1} [TopologicalSpace α] {f : α} (h₁ : Continuous f) (h₂ : ∀ (x : α), 0 < (f x).re (f x).im 0) :
    Continuous fun t => Complex.log (f t)