Derivative and series expansion of real logarithm #
In this file we prove that Real.log is infinitely smooth at all nonzero x : ℝ. We also prove
that the series ∑' n : ℕ, x ^ (n + 1) / (n + 1) converges to (-Real.log (1 - x)) for all
x : ℝ, |x| < 1.
Tags #
logarithm, derivative
A crude lemma estimating the difference between log (1-x) and its Taylor series at 0,
where the main point of the bound is that it tends to 0. The goal is to deduce the series
expansion of the logarithm, in hasSum_pow_div_log_of_abs_lt_1.
TODO: use one of generic theorems about Taylor's series to prove this estimate.
Compute the derivative of the difference between $\frac{1}{2} * \log(\frac{1+x}{1-x})$ and its
Taylor series at 0 up to order n. This is an auxiliary lemma for
sum_range_sub_log_div_le and sum_range_le_log_div.
Note that thanks to the geometric series, the derivative has a particularly simple form, and means
that it is more convenient to avoid Taylor's theorem.
A lemma estimating the difference between $\frac{1}{2} * \log(\frac{1+x}{1-x})$ and its
Taylor series at 0, where the bound tends to 0. This bound is particularly useful for explicit
estimates of logarithms.
Note that thanks to the geometric series, the derivative has a particularly simple form, and means that it is more convenient to avoid Taylor's theorem for this proof.
For 0 ≤ x < 1, the partial sums of the series expansion of $\frac{1}{2} * \log(\frac{1+x}{1-x})$
at 0 form a lower bound for it. This shows that the absolute value in sum_range_sub_log_div_le
can be dropped, and gives explicit lower bounds for logarithms.