Zulip Chat Archive
Stream: maths
Topic: Antilipschitz for linear maps
Yury G. Kudryashov (Feb 23 2025 at 21:29):
Currently, different lemmas use different spelling for the assumption "a CLM f'
is an expanding map":
- docs#HasFDerivAtFilter.isBigO_sub_rev uses
{C} (h : AntilipschitzWith C f')
; - docs#HasStrictFDerivAt.isBigO_sub_rev assumes that
f'
is an equivalence (which is stronger than what we actually need); - docs#HasFDerivWithinAt.eventually_ne assumes
∃ C, ∀ z, ‖z‖ ≤ C * ‖f' z‖
I think that we should normalize these assumptions, preferrably to something that doesn't depend on the norm, so that we can generalize to TVS later.
Yury G. Kudryashov (Feb 23 2025 at 21:32):
/poll Possible options:
id =O[⊤] f'
, then generalize to TVS using not-yet-in-mathlib IsBigOTVS
;
id =O[𝓝 0] f'
, then generalize to TVS using not-yet-in-mathlib IsBigOTVS
;
comap f (𝓝 0) ≤ 𝓝 0
new definition with constructors/lemmas linking to all other versions here.
Yury G. Kudryashov (Feb 23 2025 at 21:32):
For the comap
version see docs#LinearMap.antilipschitz_of_comap_nhds_le
Yury G. Kudryashov (Feb 23 2025 at 21:34):
The main issues with the first 2 approaches are:
- it isn't clear which one is better;
- we'll have to either redo
Is*OTVS
for different scalar fields on the LHS and RHS, or restrict this normal form to linear, not semilinear maps.
Yury G. Kudryashov (Feb 23 2025 at 21:35):
Given that we have many different options, I slightly prefer to add a new definition here.
Eric Wieser (Feb 23 2025 at 23:49):
I have repeatedly hallucinated the existence of Lipschitz
and Antilipschitz
as existentially-quantified version of the With
versions, so I would be in favor of them being introduced one way or another
Yury G. Kudryashov (Feb 24 2025 at 01:40):
We may need something LinearMap
-specific too, because we can't say Antilipschitz
without having a metric, and I want to use this as an assumption in some theorems about derivatives.
Yury G. Kudryashov (Feb 24 2025 at 01:40):
Currently, these lemmas use normed spaces, but we're going to generalize them to TVS soon.
Antoine Chambert-Loir (Feb 25 2025 at 08:48):
Isn't it strictness of the linear map? (Quotient topology coincides with the subspace topology on the range)?
Yury G. Kudryashov (Feb 25 2025 at 08:52):
Why quotient topology? This condition implies injectivity (at least, for Hausdorff spaces).
Yury G. Kudryashov (Feb 25 2025 at 08:54):
It may be equivalent to IsOpenEmbedding
(for continuous linear maps), but I'm too sleepy now to be sure.
Anatole Dedecker (Feb 27 2025 at 21:22):
Yes, nhds 0 = comap f (nhds zero)
is precisely the same as IsOpenEmbedding
as long as f
is an add group morphism between topological additive groups. This even holds under the condition that addition of any fixed constant is continuous, but there’s no hope for any of this to hold in monoids (I don’t think we care though: in any more general setup, I claim that docs#IsOpenEmbedding is obviously the right analog)
Antoine Chambert-Loir (Mar 01 2025 at 21:35):
Sorry, you're right.
Last updated: May 02 2025 at 03:31 UTC