Documentation

Mathlib.NumberTheory.Harmonic.Bounds

This file proves $\log(n+1) \le H_n \le 1 + \log(n)$ for all natural numbers $n$.

theorem harmonic_eq_sum_Icc {n : } :
harmonic n = iFinset.Icc 1 n, (↑i)⁻¹
theorem log_add_one_le_harmonic (n : ) :
Real.log ↑(n + 1) (harmonic n)