Lemmas about Nat.nthRoot
#
In this file we prove that Nat.nthRoot n a
is indeed the floor of ⁿ√a
.
TODO #
Rewrite the proof of Nat.nthRoot.lt_pow_go_succ_aux
to avoid dependencies on real numbers,
so that we can move this file to Mathlib/Data/Nat/NthRoot
, then to Batteries.
Alias of the reverse direction of Nat.pow_nthRoot_le_iff
.
nthRoot n a ^ n ≤ a
unless both n
and a
are zeros.
An auxiliary lemma saying that if b ≠ 0
,
then (a / b ^ n + n * b) / (n + 1) + 1
is a strict upper estimate on √[n + 1] a
.
Currently, the proof relies on the weighted AM-GM inequality, which increases the dependency closure of this file by a lot.
A PR proving this inequality by more elementary means is very welcome.