Zulip Chat Archive

Stream: Is there code for X?

Topic: Abel's summation and/or Stieltjes integration


Meow (Jan 12 2023 at 11:16):

Is Abel's summation and Euler-Maclaurin summation formalized in Lean? In mathlib we have Stieltjes measure (for monotone functions), and Abel's summation is just the integration by part of Stieltjes integration.

Meow (Jan 12 2023 at 11:18):

https://leanprover.zulipchat.com/#narrow/stream/116395-maths/topic/analytical.20number.20theory/near/320708370

David Loeffler (Jan 12 2023 at 11:26):

Euler-Maclaurin summation isn't in mathlib but it will be easy to add, since it doesn't need any new work on the measure-theory side.

David Loeffler (Jan 12 2023 at 11:29):

For Abel summation (assuming you mean the first statement here : https://en.wikipedia.org/wiki/Abel%27s_summation_formula), it might be easier to prove it more directly, rather than going through the work of defining the Stieltjes integral in the relevant settings.

Meow (Jan 12 2023 at 11:52):

Yes, that's my opinion.

Xavier Roblot (Nov 15 2024 at 15:22):

I have an almost complete proof of Abel summation formula (just a couple of easy sorries to fill in) but I wanted to make sure it is the right formulation / hypotheses before going further. Basically, what I have is the following:

import Mathlib

open Finset intervalIntegral MeasureTheory

variable (c :   ) (f :   )

abbrev S :    := fun t   n  range (t + 1⌋₊), c n

theorem AbelSummation {x : }
    (h_diff :  t  Set.Icc (0 : ) x, DifferentiableAt  f t)
    (h_integ : IntervalIntegrable (deriv f) volume 0 x) :
     k  range (x + 1⌋₊), c k * f k = S c x * f x -  t in (0 : )..x, S c t * deriv f t := by sorry

Ruben Van de Velde (Nov 15 2024 at 15:24):

Oh, I have a proof in PNT+

Ruben Van de Velde (Nov 15 2024 at 15:24):

https://github.com/AlexKontorovich/PrimeNumberTheoremAnd/pull/191

Xavier Roblot (Nov 15 2024 at 15:32):

Are you planning on PR'ing it soon?

Xavier Roblot (Nov 15 2024 at 15:33):

Also, you use docs#ContinuousOn and I use docs#IntervalIntegrable. One question I have is which one is better in general?

Ruben Van de Velde (Nov 15 2024 at 15:42):

I have no opinion - I just bashed out something that would work in the case I needed. I had no immediate plans to PR it to mathlib, but I can try to get around to it (or you could, if you have time)

Vincent Beffara (Nov 15 2024 at 15:42):

How far is this from docs#Finset.sum_range_by_parts plus docs#intervalIntegral.integral_deriv_eq_sub plus docs#intervalIntegral.sum_integral_adjacent_intervals ?

Xavier Roblot (Nov 15 2024 at 15:43):

Vincent Beffara said:

How far is this from docs#Finset.sum_range_by_parts plus docs#intervalIntegral.integral_deriv_eq_sub plus docs#intervalIntegral.sum_integral_adjacent_intervals ?

This is basically my proof

Xavier Roblot (Nov 15 2024 at 15:43):

It's pretty straightforward

Xavier Roblot (Nov 19 2024 at 12:30):

@Ruben Van de Velde I have a version of Abel summation here that I am reasonably happy with and I would like to PR it if you don't mind since I'll need it at some point for the proof of the analytic class number formula. It just needs a good name, a place to live and probably also some golfing

Ruben Van de Velde (Nov 19 2024 at 12:30):

No, don't mind at all

Xavier Roblot (Nov 19 2024 at 12:32):

Thanks! I'll be also very interested in your review once it's ready :wink:

Xavier Roblot (Nov 19 2024 at 12:33):

And any suggestion for names and/or location !

Ruben Van de Velde (Nov 19 2024 at 12:33):

Please ping me on zulip if you want me to review, I'm in permanent github notification bankrupcy

Kevin Buzzard (Nov 20 2024 at 07:57):

Do you want some of my notifications?

Xavier Roblot (Nov 20 2024 at 14:28):

@Ruben Van de Velde , the PR is ready: #19289


Last updated: May 02 2025 at 03:31 UTC