Comparing sums and integrals #
Summary #
It is often the case that error terms in analysis can be computed by comparing an infinite sum to the improper integral of an antitone function. This file will eventually enable that.
At the moment it contains several lemmas in this direction, for antitone or monotone functions
(or products of antitone and monotone functions), formulated for sums on range i
or Ico a b
.
TODO
: Add more lemmas to the API to directly address limiting issues
Main Results #
AntitoneOn.integral_le_sum
: The integral of an antitone function is at most the sum of its values at integer steps aligning with the left-hand side of the intervalAntitoneOn.sum_le_integral
: The sum of an antitone function along integer steps aligning with the right-hand side of the interval is at most the integral of the function along that intervalMonotoneOn.integral_le_sum
: The integral of a monotone function is at most the sum of its values at integer steps aligning with the right-hand side of the intervalMonotoneOn.sum_le_integral
: The sum of a monotone function along integer steps aligning with the left-hand side of the interval is at most the integral of the function along that intervalsum_mul_Ico_le_integral_of_monotone_antitone
: the sum off i * g i
on an interval is bounded by the integral off x * g (x - 1)
iff
is monotone andg
is antitone.integral_le_sum_mul_Ico_of_antitone_monotone
: the sum off i * g i
on an interval is bounded below by the integral off x * g (x - 1)
iff
is antitone andg
is monotone.
Tags #
analysis, comparison, asymptotics
theorem
sum_Ico_le_integral_of_le
{a b : ℕ}
{f g : ℝ → ℝ}
(hab : a ≤ b)
(h : ∀ i ∈ Set.Ico a b, ∀ x ∈ Set.Ico ↑i ↑(i + 1), f ↑i ≤ g x)
(hg : MeasureTheory.IntegrableOn g (Set.Ico ↑a ↑b) MeasureTheory.volume)
:
theorem
integral_le_sum_Ico_of_le
{a b : ℕ}
{f g : ℝ → ℝ}
(hab : a ≤ b)
(h : ∀ i ∈ Set.Ico a b, ∀ x ∈ Set.Ico ↑i ↑(i + 1), g x ≤ f ↑i)
(hg : MeasureTheory.IntegrableOn g (Set.Ico ↑a ↑b) MeasureTheory.volume)
:
theorem
AntitoneOn.integral_le_sum_Ico
{a b : ℕ}
{f : ℝ → ℝ}
(hab : a ≤ b)
(hf : AntitoneOn f (Set.Icc ↑a ↑b))
:
theorem
MonotoneOn.sum_le_integral_Ico
{a b : ℕ}
{f : ℝ → ℝ}
(hab : a ≤ b)
(hf : MonotoneOn f (Set.Icc ↑a ↑b))
: