Absolute values of complex numbers #
Absolute value #
The complex absolute value function, defined as the square root of the norm squared.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Cauchy sequences #
The real part of a complex Cauchy sequence, as a real Cauchy sequence.
Equations
- Complex.cauSeqRe f = ⟨fun (n : ℕ) => (↑f n).re, ⋯⟩
Instances For
The imaginary part of a complex Cauchy sequence, as a real Cauchy sequence.
Equations
- Complex.cauSeqIm f = ⟨fun (n : ℕ) => (↑f n).im, ⋯⟩
Instances For
The limit of a Cauchy sequence of complex numbers.
Equations
- Complex.limAux f = { re := (Complex.cauSeqRe f).lim, im := (Complex.cauSeqIm f).lim }
Instances For
theorem
Complex.isCauSeq_conj
(f : CauSeq ℂ ⇑abs)
:
IsCauSeq ⇑abs fun (n : ℕ) => (starRingEnd ℂ) (↑f n)
The complex conjugate of a complex Cauchy sequence, as a complex Cauchy sequence.
Equations
- Complex.cauSeqConj f = ⟨fun (n : ℕ) => (starRingEnd ℂ) (↑f n), ⋯⟩
Instances For
The absolute value of a complex Cauchy sequence, as a real Cauchy sequence.
Equations
- Complex.cauSeqAbs f = ⟨⇑Complex.abs ∘ ↑f, ⋯⟩