mathlib documentation

topology.instances.complex

@[instance]

Equations
theorem complex.dist_eq (x y : ) :
dist x y = complex.abs (x - y)

theorem complex.uniform_continuous_inv (s : set ) {r : } (r0 : 0 < r) (H : ∀ (x : ), x sr complex.abs x) :

theorem complex.tendsto_inv {r : } (r0 : r 0) :
(λ (q : ), q⁻¹)→_{r}r⁻¹

theorem complex.continuous_inv  :
continuous (λ (a : {r // r 0}), (a.val)⁻¹)

theorem complex.continuous.inv {α : Type u_1} [topological_space α] {f : α → } (h : ∀ (a : α), f a 0) (hf : continuous f) :
continuous (λ (a : α), (f a)⁻¹)

theorem complex.uniform_continuous_mul (s : set ( × )) {r₁ r₂ : } (H : ∀ (x : × ), x scomplex.abs x.fst < r₁ complex.abs x.snd < r₂) :
uniform_continuous (λ (p : s), (p.val.fst) * p.val.snd)

theorem complex.continuous_mul  :
continuous (λ (p : × ), (p.fst) * p.snd)

is homeomorphic to the real plane with max norm.

Equations