Documentation

Mathlib.Data.Complex.Norm

Norm on the complex numbers #

Equations
@[simp]
theorem Complex.norm_eq_abs (z : ) :
Equations
  • One or more equations did not get rendered due to their size.
theorem Complex.dist_eq (z w : ) :
dist z w = abs (z - w)
theorem Complex.dist_eq_re_im (z w : ) :
dist z w = ((z.re - w.re) ^ 2 + (z.im - w.im) ^ 2)
@[simp]
theorem Complex.dist_mk (x₁ y₁ x₂ y₂ : ) :
dist { re := x₁, im := y₁ } { re := x₂, im := y₂ } = ((x₁ - x₂) ^ 2 + (y₁ - y₂) ^ 2)
theorem Complex.dist_of_re_eq {z w : } (h : z.re = w.re) :
dist z w = dist z.im w.im
theorem Complex.nndist_of_re_eq {z w : } (h : z.re = w.re) :
nndist z w = nndist z.im w.im
theorem Complex.edist_of_re_eq {z w : } (h : z.re = w.re) :
edist z w = edist z.im w.im
theorem Complex.dist_of_im_eq {z w : } (h : z.im = w.im) :
dist z w = dist z.re w.re
theorem Complex.nndist_of_im_eq {z w : } (h : z.im = w.im) :
nndist z w = nndist z.re w.re
theorem Complex.edist_of_im_eq {z w : } (h : z.im = w.im) :
edist z w = edist z.re w.re
@[simp]
theorem Complex.norm_real (r : ) :
@[simp]
theorem Complex.norm_natCast (n : ) :
n = n
@[simp]
theorem Complex.norm_intCast (n : ) :
n = |n|
@[simp]
theorem Complex.norm_ratCast (q : ) :
q = |q|
@[simp]
@[simp]
theorem Complex.nnnorm_natCast (n : ) :
n‖₊ = n
@[simp]
@[deprecated Complex.norm_natCast (since := "2024-08-25")]
theorem Complex.norm_nat (n : ) :
n = n

Alias of Complex.norm_natCast.

@[deprecated Complex.norm_intCast (since := "2024-08-25")]
theorem Complex.norm_int (n : ) :
n = |n|

Alias of Complex.norm_intCast.

@[deprecated Complex.norm_ratCast (since := "2024-08-25")]
theorem Complex.norm_rat (q : ) :
q = |q|

Alias of Complex.norm_ratCast.

@[deprecated Complex.nnnorm_natCast (since := "2024-08-25")]
theorem Complex.nnnorm_nat (n : ) :
n‖₊ = n

Alias of Complex.nnnorm_natCast.

@[simp]
theorem Complex.norm_nnratCast (q : ℚ≥0) :
q = q
@[simp]
theorem Complex.norm_int_of_nonneg {n : } (hn : 0 n) :
n = n