@@ -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
534540This 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
539545Several properties of the sum transform are then proven.
540546-/
0 commit comments