Zulip Chat Archive

Stream: Is there code for X?

Topic: Roughly, Lipschitzness of the inverse of `exp (t * I)`


Geoffrey Irving (Feb 18 2024 at 14:25):

Do we have this, or something which can easily get to it:

import Mathlib.Analysis.SpecialFunctions.Trigonometric.Basic
open Complex (abs exp I)
open scoped Real

lemma lipschitz_inv_exp_mul_I {t : } (m : t  Set.Ioc (-π) π) :
    |t|  π / 2 * abs (exp (t * I) - 1) := by
  sorry

Geoffrey Irving (Feb 18 2024 at 14:28):

It's equivalent to t^2 ≤ π^2/2 * (1 - cos t).

Yaël Dillies (Feb 18 2024 at 14:34):

I just proved this in a PR

Yaël Dillies (Feb 18 2024 at 14:35):

I needed to show the arc-distance and chord distance on the circle are equivalent

Geoffrey Irving (Feb 18 2024 at 14:35):

Yes, that’s also why I need it.

Geoffrey Irving (Feb 18 2024 at 14:35):

Which PR?

Yaël Dillies (Feb 18 2024 at 14:35):

#10226

Geoffrey Irving (Feb 18 2024 at 14:37):

Thanks! I will steal it for now with comments to strip it once it’s in.

Geoffrey Irving (Feb 18 2024 at 14:40):

Actually might just leave mine as sorry, as it’ll probably be in before I finish the rest of Koebe.

Yaël Dillies (Feb 18 2024 at 14:41):

(best way to make sure it's in is to review it :pray:)

Geoffrey Irving (Feb 18 2024 at 14:44):

Happy to! Anything I need to do prior to that, or should I just do it now? (Might end up as this evening.)

Yaël Dillies (Feb 18 2024 at 14:56):

Nothing to do prior to that. Anybody can review anything anytime

Eric Wieser (Feb 18 2024 at 14:58):

There is a review guide at https://leanprover-community.github.io/contribute/pr-review.html, which has lots of Lean-specific advice even if you're no stranger to code review.

Geoffrey Irving (Feb 18 2024 at 15:08):

Great, will read through that and review this evening.

Geoffrey Irving (Feb 18 2024 at 15:09):

Though there are already several reviewers? Not sure what the norms are in such situations.

Jireh Loreaux (Feb 18 2024 at 15:11):

You're always welcome to add your review, regardless of who else has reviewed.

Jireh Loreaux (Feb 18 2024 at 15:12):

Of course, you may want to read through what prior reviews have said so you don't duplicate.

Geoffrey Irving (Feb 18 2024 at 21:42):

"Approved", FWIW. But to check: where is the result I wanted in that PR? Is it elsewhere in the angle theory, and now there's a bridge between the two?

Yaël Dillies (Feb 18 2024 at 22:02):

Whoops sorry I meant #10525, not #10226

Yaël Dillies (Feb 18 2024 at 22:02):

Seems like my clipboard played me

Geoffrey Irving (Feb 18 2024 at 22:03):

I'll review that one too in a moment.


Last updated: May 02 2025 at 03:31 UTC