Skip to content

Commit ceb11f3

Browse files
committed
doc(AkraBazzi): minor tweaks and additions (#30499)
Broken out of #29464 to simplify review. This PR: - Makes the implementation note in GrowsPolynomially.lean more concise. - Expands the "Main definitions and results" section in SumTransform.lean
1 parent d4c295d commit ceb11f3

File tree

2 files changed

+19
-13
lines changed

2 files changed

+19
-13
lines changed

Mathlib/Computability/AkraBazzi/GrowsPolynomially.lean

Lines changed: 5 additions & 5 deletions
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ import Mathlib.Algebra.Order.ToIntervalMod
1010
import Mathlib.Analysis.SpecialFunctions.Log.Base
1111

1212
/-!
13-
# Akra-Bazzi theorem: The polynomial growth condition
13+
# Akra-Bazzi theorem: the polynomial growth condition
1414
1515
This file defines and develops an API for the polynomial growth condition that appears in the
1616
statement of the Akra-Bazzi theorem: for the theorem to hold, the function `g` must
@@ -19,10 +19,10 @@ satisfy the condition that `c₁ g(n) ≤ g(u) ≤ c₂ g(n)`, for u between b*n
1919
2020
## Implementation notes
2121
22-
Our definition requires that the condition must hold for any `b ∈ (0,1)`. This is equivalent to
23-
requiring it for `b = 1 / 2` (or any other particular value in `(0, 1)`). While this could, in
24-
principle, make it harder to prove that a particular function grows polynomially, this issue does
25-
not seem to arise in practice.
22+
Our definition requires that the condition hold for any `b ∈ (0,1)`. This is equivalent to requiring
23+
it only for `b = 1 / 2` (or any other particular value in `(0, 1)`). While this could, in principle,
24+
make it harder to prove that a particular function grows polynomially, this issue does not seem to
25+
arise in practice.
2626
2727
-/
2828

Mathlib/Computability/AkraBazzi/SumTransform.lean

Lines changed: 14 additions & 8 deletions
Original file line numberDiff line numberDiff line change
@@ -17,11 +17,17 @@ We develop further preliminaries required for the theorem, up to the sum transfo
1717
## Main definitions and results
1818
1919
* `AkraBazziRecurrence T g a b r`: the predicate stating that `T : ℕ → ℝ` satisfies an Akra-Bazzi
20-
recurrence with parameters `g`, `a`, `b` and `r` as above.
21-
* `sumTransform`: The transformation which turns a function `g` into
22-
`n^p * ∑ u ∈ Finset.Ico n₀ n, g u / u^(p+1)`.
23-
* `asympBound`: The asymptotic bound satisfied by an Akra-Bazzi recurrence, namely
24-
`n^p (1 + ∑ g(u) / u^(p+1))`
20+
recurrence with parameters `g`, `a`, `b` and `r` as above, together with basic bounds on `r i n`
21+
and positivity of `T`.
22+
* `AkraBazziRecurrence.smoothingFn`: the smoothing function $\varepsilon(x) = 1 / \log x$ used in
23+
the inductive estimates, along with monotonicity, differentiability, and asymptotic properties.
24+
* `AkraBazziRecurrence.p`: the unique Akra–Bazzi exponent characterized by $\sum_i a_i\,(b_i)^p = 1`
25+
and supporting analytical lemmas such as continuity and injectivity of the defining sum.
26+
* `AkraBazziRecurrence.sumTransform`: the transformation that turns a function `g` into
27+
`n^p * ∑ u ∈ Finset.Ico n₀ n, g u / u^(p+1)` and its eventual comparison with multiples of `g n`.
28+
* `AkraBazziRecurrence.asympBound`: the asymptotic bound satisfied by an Akra-Bazzi recurrence,
29+
namely `n^p (1 + ∑ g(u) / u^(p+1))`, together with positivity statements along the branches
30+
`r i n`.
2531
2632
2733
## References
@@ -532,9 +538,9 @@ lemma sumCoeffsExp_p_eq_one : ∑ i, a i * (b i) ^ p a b = 1 := by
532538
### The sum transform
533539
534540
This section defines the "sum transform" of a function `g` as
535-
`∑ u ∈ Finset.Ico n₀ n, g u / u^(p+1)`, and uses it to define `asympBound` as the bound satisfied
536-
by an Akra-Bazzi recurrence, namely `n^p (1 + ∑_{u < n} g(u) / u^(p+1))`. Here, the exponent `p`
537-
refers to the one established in the previous section.
541+
`∑ u ∈ Finset.Ico n₀ n, g u / u ^ (p + 1)`, and uses it to define `asympBound` as the bound
542+
satisfied by an Akra-Bazzi recurrence, namely `n^p (1 + ∑_{u < n} g(u) / u^(p+1))`. Here, the
543+
exponent `p` refers to the one established in the previous section.
538544
539545
Several properties of the sum transform are then proven.
540546
-/

0 commit comments

Comments
 (0)