Estimates for the complex logarithm #
We show that log (1+z)
differs from its Taylor polynomial up to degree n
by at most
‖z‖^(n+1)/((n+1)*(1-‖z‖))
when ‖z‖ < 1
; see Complex.norm_log_sub_logTaylor_le
.
To this end, we derive the representation of log (1+z)
as the integral of 1/(1+tz)
over the unit interval (Complex.log_eq_integral
) and introduce notation
Complex.logTaylor n
for the Taylor polynomial up to degree n-1
.
TODO #
Refactor using general Taylor series theory, once this exists in Mathlib.
Integral representation of the complex log #
The Taylor polynomials of the logarithm #
The n
th Taylor polynomial of log
at 1
, as a function ℂ → ℂ
Equations
- Complex.logTaylor n z = ∑ j ∈ Finset.range n, (-1) ^ (j + 1) * z ^ j / ↑j
Instances For
theorem
Complex.hasDerivAt_logTaylor
(n : ℕ)
(z : ℂ)
:
HasDerivAt (logTaylor (n + 1)) (∑ j ∈ Finset.range n, (-1) ^ j * z ^ j) z