Zulip Chat Archive

Stream: Is there code for X?

Topic: Topological sums and complex powers


Michael Stoll (Mar 12 2024 at 19:39):

I'm trying to produce a proof of

import Mathlib

open LSeries Complex

open Filter in
lemma LSeries_limit {f :   } {n : } (h :  m  n, f m = 0) (ha : abscissaOfAbsConv f < ):
    Tendsto (fun x :   ((n + 1) ^ (x : )) * LSeries f x) atTop (nhds (f (n + 1))) := sorry

(which is the main ingredient to then prove

/-- The `LSeries` of `f` is zero if and only if either `f = 0`
or the L-series converges nowhere. -/
lemma LSeries_eq_zero_iff {f :   } (hf : f 0 = 0) :
    LSeries f = 0  f = 0  abscissaOfAbsConv f =  := sorry

from which it easily follows that a converging L-series determines its coefficients).

But I find it very painful.

One problem I managed to solve, but with a rather ugly proof, is

import Mathlib

example (m n : ) (z : ) (x : ) :
    (n + 1) ^ (x : ) * (z / m ^ (x : )) = z / (m / (n + 1)) ^ (x : ) := by
  sorry

Am I missing something here?

Another thing that would be helpful is a version of docs#tendsto_tsum_of_dominated_convergence where the bound needs to hold only eventually instead of everywhere.

Michael Stoll (Mar 12 2024 at 19:45):

E.g., I can do this:

import Mathlib

open Filter in
lemma foo {f :     } {x : } (hx : Summable (f x)) (hb :  y  x,  n, f y n  f x n)
    (hc :  n, Tendsto (f · n) atTop (nhds 0)) :
    Tendsto (fun x  tsum (f x)) atTop (nhds 0) := by
  rw [show (0 : ) = tsum (fun _ :   0) by simp]
  refine tendsto_tsum_of_dominated_convergence hx.norm hc fun y n  hb y ?_ n
  -- stuck here, goal is `y ≥ x`
  sorry

Terence Tao (Mar 12 2024 at 20:27):

One can split the L-series in the regimes m(n+1)2m \leq (n+1)^2 and m>(n+1)2m > (n+1)^2. The first regime is a finite sum and should be straightforward. For the tail, use (n+1)x/mx1/mx/2 (n+1)^{x} / m^{x} \leq 1 / m^{x/2} to get domination once xx is non-negative and also at least twice the abscissa of convergence.

Michael Stoll (Mar 12 2024 at 20:44):

This does not solve the problem since the result that is in Mathlib requires to show the bound for all xx. Your argument still imposes a lower bound on xx.

Michael Stoll (Mar 12 2024 at 20:46):

I can probably work around that by using a piecewise defined function that is zero when y < x (using notation as in foo above) and equal to f otherwise, applying docs#tendsto_tsum_of_dominated_convergence to that, and using a suitable congruence lemma (that reduces to eventual equality). But this is a bit ugly...

Anatole Dedecker (Mar 12 2024 at 22:25):

Would #11236 solve your issues ?

Eric Wieser (Mar 12 2024 at 22:51):

(just sent that one to bors, since it had David's backing and the code looks fine)

Michael Stoll (Mar 13 2024 at 10:56):

Thanks! This is exeactly what I need for this part of the problem.


Last updated: May 02 2025 at 03:31 UTC