Zulip Chat Archive

Stream: condensed mathematics

Topic: profinite trivialities


Johan Commelin (Apr 10 2021 at 05:45):

https://github.com/leanprover-community/lean-liquid/blob/master/src/pseudo_normed_group/FiltrationPow.lean#L69 defines Pow which takes powers of profinite sets.

  • We'll need Pow_mul and Pow_mul' which give functorial isos Xmn(Xm)nXnmX^{mn} \cong (X^m)^n \cong X^{nm}.
  • Do we already have iso_of_homeomorph for Profinite?

Adam Topaz (Apr 10 2021 at 13:06):

In the cech_stuff branch, I added iso_of_bijective :wink:

Filippo A. E. Nuccio (Apr 22 2022 at 14:52):

I am trying to prove that a certain set is open in the space of bounded Laurent measures. If I look at these as a "honest" inverse limit, I know how to do, because my set is a product of some subsets of finitely many components, and then the whole component elsewhere, using docs#topological_space.is_topological_basis.is_open_iff . I also get that the topology on the bounded Laurent measures is induced from that on the limit cone (the two types are equivalent), and I wonder if there is a painless way to describe this limit cone as a subtype of the Pi type.

Johan Commelin (Apr 22 2022 at 14:56):

There is a homeomorphism between the two. I'm not near Lean right now, but it should be somewhere close to the definition of the topology.

Filippo A. E. Nuccio (Apr 22 2022 at 14:57):

Well, I can find laurent_measures_bdd_homeo { F : ℒ S | ∥F∥₊ ≤ c } ≃ₜ (Profinite.limit_cone (laurent_measures_bdd_functor r S c ⋙ Fintype.to_Profinite)).X, is it the one you are referring to?

Filippo A. E. Nuccio (Apr 22 2022 at 14:58):

This is actually not very useful, I think: it is basically tautological, because the topology on laurent measures is defined as the topology on the limit cone.

Adam Topaz (Apr 22 2022 at 15:00):

@Filippo A. E. Nuccio Are you working with a subset of one of the filtered pieces of Laurent measures? I suppose so, because otherwise there is no topology!

Filippo A. E. Nuccio (Apr 22 2022 at 15:01):

Yes, indeed.

Adam Topaz (Apr 22 2022 at 15:01):

Note that Profinite.limit_cone is defeq to the "usual" limit, i.e. as a closed subset of the pi type

Filippo A. E. Nuccio (Apr 22 2022 at 15:01):

Really defeq?!

Adam Topaz (Apr 22 2022 at 15:01):

Yeah, it should be

Adam Topaz (Apr 22 2022 at 15:02):

https://github.com/leanprover-community/mathlib/blob/631890bf90e76818b80c57c00291380c0329143d/src/topology/category/Profinite/default.lean#L161

Filippo A. E. Nuccio (Apr 22 2022 at 15:02):

Wow, so I can blindly apply your result on the basis of the topology of a Pi.top space and get somewhere? I did not even dare trying... :smiling_face:

Filippo A. E. Nuccio (Apr 22 2022 at 15:02):

Adam Topaz said:

https://github.com/leanprover-community/mathlib/blob/631890bf90e76818b80c57c00291380c0329143d/src/topology/category/Profinite/default.lean#L161

Oh nice!

Filippo A. E. Nuccio (Apr 22 2022 at 15:02):

Thanks

Adam Topaz (Apr 22 2022 at 15:02):

well, first you apply ssome lemma about the induced topology

Filippo A. E. Nuccio (Apr 22 2022 at 15:03):

Yes yes, this I thought.

Adam Topaz (Apr 22 2022 at 15:03):

since you need to pass from the subspace to the ambient pi type

Adam Topaz (Apr 22 2022 at 15:03):

It all boils down to the following construction
https://github.com/leanprover-community/mathlib/blob/631890bf90e76818b80c57c00291380c0329143d/src/topology/category/Top/limits.lean#L40

Filippo A. E. Nuccio (Apr 22 2022 at 15:03):

OK, I will try but it seems easy, thanks.

Adam Topaz (Apr 22 2022 at 15:06):

If you want, there is also docs#Top.limit_cone_infi which you can use in conjunction with the fact that Profinite_to_Top preserves limits to obtain a description of the limit Profinite set as the infimum of topologies. IIRC I also proved some lemma (in mathlib?) describing a basis for the topology of an infimum of topologies.

Adam Topaz (Apr 22 2022 at 15:07):

docs#is_topological_basis_infi

Filippo A. E. Nuccio (Apr 22 2022 at 15:07):

Thanks, I think the lemmas about explicit Pi topologies (rather than general infi ones) should be enough, but if not I'll try these.

Kevin Buzzard (Apr 22 2022 at 15:56):

Filippo -- if you're talking about what I think you're talking about, then maybe it's enough to observe that the profinite thing you have is defined as a limit, so there will be map to one of the factors (all of which are finite), and this map will be known to be continuous, and then you can take the preimage of a point in the factor and this will be open.

Filippo A. E. Nuccio (Apr 22 2022 at 15:57):

Oh, very good point Kevin. I am indeed talking about what I think you think I am talking about... :sweat_smile:

Filippo A. E. Nuccio (Apr 22 2022 at 15:59):

I am grabbing this option to dwell a bit into the category_theory library, and construction of limits, but I will probably take your approach soon.

Filippo A. E. Nuccio (Apr 22 2022 at 15:59):

Thanks.


Last updated: Dec 20 2023 at 11:08 UTC