Documentation

Mathlib.Analysis.Complex.CoveringMap

Covering maps involving the complex plane #

In this file, we show that Complex.exp is a covering map on {0}ᶜ.

exp : ℂ → ℂ \ {0} is a covering map.

theorem Polynomial.isCoveringMapOn_eval {𝕜 : Type u_1} [NontriviallyNormedField 𝕜] [ProperSpace 𝕜] (p : Polynomial 𝕜) :
IsCoveringMapOn (fun (x : 𝕜) => eval x p) ((fun (x : 𝕜) => eval x p) '' {k : 𝕜 | eval k (derivative p) = 0})