Zulip Chat Archive

Stream: Is there code for X?

Topic: 1/(n+1) is decreasing


Michael Stoll (Feb 22 2024 at 10:59):

Looking for

import Mathlib

example : Antitone (fun n :   (n + 1 : )⁻¹) := sorry

but having problems finding it in Mathlib...

@loogle Antitone, Inv.inv

loogle (Feb 22 2024 at 10:59):

:search: Antitone.inv, Monotone.inv, and 1 more

Eric Rodriguez (Feb 22 2024 at 12:20):

example : Antitone (fun n :   (n + 1 : )⁻¹) := by
  intros a b h
  apply inv_le_inv_of_le
  · positivity
  gcongr

Eric Rodriguez (Feb 22 2024 at 12:20):

but inv_0 lemmas are lacking...

Michael Stoll (Feb 22 2024 at 12:26):

Thanks; I had a similar proof.
The real question is, I guess, whether some form of this should be in Mathlib.

Damiano Testa (Feb 22 2024 at 12:29):

Btw, there is a current thread with a similar problem of missing inv\0 lemmas.

I personally would expect the inv\0 lemmas to exist.

Michael Stoll (Feb 22 2024 at 12:33):

There is docs#inv_le_inv₀, but it only applies to a LinearOrderedCommGroupWithZero, which I think the reals are not.

Kevin Buzzard (Feb 22 2024 at 12:36):

Yeah I think that's for general valuation theory, which demands that 0 is the smallest element. Can I interest you in NNReal?

Michael Stoll (Feb 22 2024 at 12:37):

Un-#xy: I need this for

lemma not_summable_indicator_one_div_natCast {m : } (hm : m  0) (k : ZMod m) :
    ¬ Summable (Set.indicator {n :  | (n : ZMod m) = k} fun n :   (1 / n : )) := sorry

which I use in turn to show that Dirichlet L-series have absicssa of absolute convergence equal to 1.
Going via NNReal looks like a significant detour here.

Arend Mellendijk (Feb 22 2024 at 13:33):

I have some antitoneOn lemmas for invat #9984, but they might be a bit of a hassle to use here.

Kevin Buzzard (Feb 23 2024 at 07:46):

Just out of interest, why do we care that the abscissa of absolute convergence is equal to one? (Other than the "because it's there" reason). Presumably for all applications it suffices to know that it's at most 1?

Michael Stoll (Feb 23 2024 at 10:43):

I think "because it's there" is a sufficient reason! :smile:


Last updated: May 02 2025 at 03:31 UTC