Zulip Chat Archive

Stream: mathlib4

Topic: Topology on Lp


Yury G. Kudryashov (Aug 28 2023 at 23:56):

In #6839, I define a UniformSpace structure on docs#MeasureTheory.Lp for all p. The goal is to port lemmas from ∀ ε > 0, ∃ f, P f ∧ snorm (f - g) < ε to Dense {f : Lp E p μ | P f}, though I postpone this to a later PR.

Yury G. Kudryashov (Aug 29 2023 at 00:01):

Since Lp does not satisfy the triangle inequality for 0 < p < 1, I had to repeat some lemmas for Lp.

Yury G. Kudryashov (Aug 29 2023 at 00:01):

I didn't add more typeclasses because we don't have more examples.

Antoine Chambert-Loir (Aug 30 2023 at 06:33):

Mathlib doesn't know about this weaker version of metric spaces where d(x,y) <= c (d(x,z)+ d(y,z)) for some constant c ?

Jireh Loreaux (Aug 30 2023 at 12:28):

Correct. We don't currently have a type class for that. However, in various places, including Lp, we have designed things in such a way that it should be possible to easily make instances of this type class once it's defined.

Filippo A. E. Nuccio (Aug 30 2023 at 14:07):

With @Heather Macbeth we made some progress in that direction in https://github.com/leanprover-community/mathlib/tree/lp_p_le_one but this has never been pushed to mathlib (and never translated into Lean4).

Yury G. Kudryashov (Aug 31 2023 at 05:39):

I'm going to add typeclasses for that. How should I call it?

Jireh Loreaux (Aug 31 2023 at 05:46):

The terminology I'm familiar with is quasi-metric and quasi-norm. I think the latter is unambiguous, but the former I think may have other meanings.

Jireh Loreaux (Aug 31 2023 at 05:56):

Indeed, Wikipedia seems to agree with my assessment. I would vote for "quasi" in both settings for consistency.

Yury G. Kudryashov (Aug 31 2023 at 06:00):

Should it be PseudoQuasiEMetricSpace or QuasiPseudoEMetricSpace?

Anatole Dedecker (Aug 31 2023 at 15:41):

Wouldn't it be more useful to give up on homogeneity but keep subadditivity? If we use fp=fp\Vert f\Vert_p = \int \vert f\vert^p for p<1p < 1 we still have a metric structure right?

Yury G. Kudryashov (Aug 31 2023 at 16:38):

Either way works for me...

Yury G. Kudryashov (Aug 31 2023 at 16:40):

@Sebastien Gouezel @Jireh Loreaux What do you think?

Sebastien Gouezel (Aug 31 2023 at 16:49):

I don't have a well-informed opinion here. The book on F-spaces that Filippo pointed to uses the homogeneous norm, but also the distance which satisfies the triangular inequality (which is not given directly by the norm, but rather a power of it). It proves that given any quasi-distance, there exists a true distance defining the same topology.

Yury G. Kudryashov (Aug 31 2023 at 16:50):

My only goal is to reformulate our "dense" lemmas in terms of docs#Dense in Lp.

Kevin Buzzard (Aug 31 2023 at 18:09):

p-Banach spaces (usual axioms for Banach space except for λv=λpv||\lambda v||=|\lambda|^p||v|| ) are all over the liquid Tensor experiment.

Yury G. Kudryashov (Aug 31 2023 at 18:38):

So, should I change the definition of snorm?

Jireh Loreaux (Aug 31 2023 at 18:44):

Yeah, I'm not sure which is preferable.

Yury G. Kudryashov (Aug 31 2023 at 18:48):

For me, it's easier to change snorm and reuse NormedAddCommGroup than to add QuasiMetricSpaces etc. So, unless someone tells me that QuasiMetricSpaces are a much better approach to LpL^p, 0<p<10<p<1, then I'll change snorm.

Adam Topaz (Aug 31 2023 at 20:35):

FWIW, here's LTE's p\ell^p as a pp-Banach space:
https://github.com/leanprover-community/lean-liquid/blob/master/src/pBanach/lp.lean

I haven't followed the discussion above, but just wanted to mention it, in case it's helpful at all.

Yury G. Kudryashov (Aug 31 2023 at 20:37):

But it's a p-Banach space for all p.

Yury G. Kudryashov (Aug 31 2023 at 20:38):

Not only for p < 1.

Yury G. Kudryashov (Aug 31 2023 at 20:38):

I mean, in that file.

Yury G. Kudryashov (Aug 31 2023 at 20:38):

BTW, is it a metric for p > 1?

Adam Topaz (Aug 31 2023 at 20:52):

https://github.com/leanprover-community/lean-liquid/blob/92f188bd17f34dbfefc92a83069577f708851aec/src/pBanach/lp.lean#L39

Adam Topaz (Aug 31 2023 at 20:55):

Looks like we used docs3#nnreal.rpow_add_le_add_rpow for the triangle inequality

Yury G. Kudryashov (Aug 31 2023 at 21:28):

So, I'll use that formula for 0 < p < 1 and the usual formula for 1 ≤ p.

Antoine Chambert-Loir (Sep 01 2023 at 16:52):

I am not sure all the intermediate categories (where various restrictions are made regarding the “distance”) are really worthy of introduction. However, a general lemma which can be found in Bourbaki (General Topology, chapter 9, §1) describes the functions d ⁣:X×X[0;+] d \colon X \times X \to [0;+\infty] such that the preimages of the intervals [0;a] [0;a] , for a>0 a >0 , generate a fundamental systems of entourages of a uniform structure. My feeling is that this lemma could be introduced, together with a name for these functions as well as a process of creation of the according uniform structure.

Antoine Chambert-Loir (Sep 01 2023 at 16:53):

image.png
(The exercise, in French… )

Antoine Chambert-Loir (Sep 01 2023 at 16:54):

and in English
image.png

Anatole Dedecker (Sep 02 2023 at 09:53):

We have docs#UniformSpace.ofFun, but not much API for it

Anatole Dedecker (Sep 02 2023 at 09:54):

Oh and it’s still too strong

Filippo A. E. Nuccio (Sep 04 2023 at 14:42):

Yury G. Kudryashov said:

So, I'll use that formula for 0 < p < 1 and the usual formula for 1 ≤ p.

This was the approach that we took with Heather.

Filippo A. E. Nuccio (Sep 04 2023 at 14:48):

Yury G. Kudryashov said:

Should it be PseudoQuasiEMetricSpace or QuasiPseudoEMetricSpace?

I have also seen the comment

Registering this separately allows for a future emetric-like structure on `PiLp p β` for `p < 1`
satisfying a relaxed triangle inequality. The terminology for this varies throughout the
literature, but it is sometimes called a *quasi-metric* or *semi-metric*. -/

on line 127 of Mathlib/Analysis/NormedSpace/PiLp.lean

Yury G. Kudryashov (Nov 02 2023 at 01:08):

I'm going to finally implement this change (redefine norm on Lp for p < 1). I have one last question: for p = 0, the formula for p < 1 gives the measure of the indicator. Does it make sense to redefine Lp 0 norm this way (currently it's just zero)?

Yury G. Kudryashov (Nov 02 2023 at 01:28):

I mean, it gives more information about f than just constant zero, so unless it breaks some useful statement, I'm going to do it.

Jireh Loreaux (Nov 02 2023 at 02:33):

Yes, I would do that. It would match PiLp and lp that way.

Yury G. Kudryashov (Nov 02 2023 at 03:35):

UPD: no, the formula gives μ univ. I'll need to override for p = 0.


Last updated: Dec 20 2023 at 11:08 UTC