Zulip Chat Archive

Stream: Is there code for X?

Topic: category of pro-objects


Kevin Buzzard (Mar 30 2023 at 14:43):

I just searched for this and there are several instances of people saying "we need the category of pro-objects" but I never found any evidence that anyone had actually made it, either in mathlib or LTE. Is it there and I missed it, or is it still not there? I need it :-) (for a student)

Adam Topaz (Mar 30 2023 at 14:48):

It’s not there

Kevin Buzzard (Mar 30 2023 at 14:48):

Thanks for putting me out of my misery :-)

Adam Topaz (Mar 30 2023 at 14:50):

@Bhavik Mehta was working on it at one point (by viewing it as a subcategory of the category of presheaves) but I don’t think it was ever completed. It’s definitely something we should have. In LTE we had a special case that roughly worked for Profinite sets as if it was Pro(Finite), but we only developed the minimal API that was needed

Kevin Buzzard (Mar 30 2023 at 16:49):

I want Pro(Artin local O-algebras with residue field k), for O some Noetherian local ring with residue field k.

Adam Topaz (Mar 30 2023 at 16:56):

Schlessinger's criterion eh?

Yaël Dillies (Mar 30 2023 at 16:57):

@Paul Lezeau? :eyes:

Paul Lezeau (Mar 30 2023 at 17:02):

@Yaël Dillies Hm I haven't written that yet but I am hoping to formalize it as soon as I'm done with exams

Kevin Buzzard (Mar 30 2023 at 17:13):

You're going to be at Imperial next year, right? That'll be interesting.

Paul Lezeau (Mar 30 2023 at 19:29):

That's the plan!

Paul Lezeau (Mar 30 2023 at 19:32):

I'm hoping to take the number theory/ geometry formalisation course if it runs next year;)

Markus Himmel (Mar 31 2023 at 05:50):

I wrote down the definition (or more precisely its dual) at branch#ind_object last year, but I felt that there are quite a few things missing about limits and Yoneda before it really makes sense to talk about the categories of ind-objects and pro-objects. I was working with the book "Categories and Sheaves" by Kashiwara and Schapira.

Reid Barton (Mar 31 2023 at 06:35):

There are several ways to construct the ind- (or pro-) completion. Kevin what do you need specifically about it? You might just write down the API you need as constant/axioms and leave it to others (or yourself) to construct later

Kevin Buzzard (Mar 31 2023 at 06:54):

I wanted (by which I mean a student of mine wanted) to state various criteria for functors coming from deformation theory of Galois representations to be representable

Adam Topaz (Mar 31 2023 at 12:24):

Prorepresentability is also important for things like étale fundamental groups. We should probably develop a general API for such things

Matthew Ballard (Mar 31 2023 at 12:28):

I just looked at the definition of power series

Adam Topaz (Mar 31 2023 at 12:33):

What do you mean?

Matthew Ballard (Mar 31 2023 at 12:45):

Given this discussion, I was curious if/how formal power series were defined.

Kevin Buzzard (Mar 31 2023 at 12:48):

Bet it's just nat -> R

Adam Topaz (Mar 31 2023 at 13:01):

Yeah that’s essentially it

Adam Topaz (Mar 31 2023 at 13:02):

And I think we’re missing the connection with the adic completion of a polynomial ring

Matthew Ballard (Mar 31 2023 at 13:04):

It laments this in the doc string

Adam Topaz (Mar 31 2023 at 13:05):

docs#power_series

Matthew Ballard (Mar 31 2023 at 13:07):

Once I-adic completion (topological or algebraic) is available it should not be hard to fill in the details.

Kevin Buzzard (Mar 31 2023 at 14:10):

I think I-adic (that's II-adic, not \ell-adic I guess) completion is now available? Or am I being over-optimistic?

Adam Topaz (Mar 31 2023 at 14:13):

docs#adic_completion

Adam Topaz (Mar 31 2023 at 14:14):

@Coleton Kotch you might be interested in this discussion

Christian Merten (Mar 24 2024 at 22:06):

@Markus Himmel: Do you have further plans with ind objects?

In particular (that's why I am reopening this old thread), have you thought about the best way to dualise docs#CategoryTheory.Limits.IndObjectPresentation to pro objects? I would like it to look like this:

import Mathlib.CategoryTheory.Limits.Indization.IndObject

universe v u

open CategoryTheory Limits

variable {C : Type u} [Category.{v} C]

structure ProObjectPresentation (A : C  Type v) where
  I : Type v
  [ : SmallCategory I]
  [hI : IsFiltered I]
  F : I  Cᵒᵖ
  ι : F  coyoneda  (Functor.const I).obj A
  isColimit : IsColimit (Cocone.mk A ι)

This should be the FGA definition. In particular it is about covariant functors, while in Kashiwara-Shapira pro-objects are defined as a subcategory of contravariant functors (i.e. presheaves). Are you okay with this?

Second question: I need a pro-yoneda lemma, i.e. given an inverse system X~=(Xi)iI\tilde X = (X_i)_{i \in I} of objects in a category C\mathcal{C}, denote by hX~h_{\tilde X} the induced functor C(Sets)\mathcal{C} \to (Sets) sending YY to limiHomC(Xi,Y)\varinjlim_{i} \mathrm{Hom}_{\mathcal{C}}(X_i, Y). Then Hom(hX~,F)limiF(Xi)\mathrm{Hom}(h_{\tilde X}, F) \cong \varprojlim_{i} F(X_i). Are you working on something related? If no, I'll start doing it.

Kevin Buzzard (Mar 24 2024 at 22:12):

If you want a test case, then I'm very interested in deforming a representation GGL2(k)G\to GL_2(k) (kk a perfect field of characteristic pp) to the category of Artin local W(k)W(k)-algebras with residue field kk...

Christian Merten (Mar 24 2024 at 22:20):

Kevin Buzzard said:

If you want a test case, then I'm very interested in deforming a representation GGL2(k)G\to GL_2(k) (kk a perfect field of characteristic pp) to the category of Artin local W(k)W(k)-algebras with residue field kk...

If I knew what that means, I would be happy to try ;-)

Kevin Buzzard (Mar 24 2024 at 22:25):

Mazur introduced, and Wiles used to great effect, this idea. If kk is a finite field then one can consider the category of commutative rings RR which are finite (as sets), local (i.e. have a unique maximal ideal mm) and have a fixed identification R/m=kR/m=k. Given a group homomorphism ρ:GGLn(k)\rho:G\to GL_n(k) we could define a lift of ρ\rho to RR to be a homomorphism ρ~:GGLn(R)\tilde\rho:G\to GL_n(R) which reduces mod mm to ρ\rho. Mazur observed that under some mild hypotheses on GG, this functor was prorepresentable, and raised the question that if GG was a Galois group and ρ\rho came from some arithmetical situation (e.g. the pp-torsion in an elliptic curve) then perhaps the prorepresenting object was arithmetically significant. Wiles showed that it was isomorphic to a Hecke algebra, and FLT followed. I'm going to need all of this machinery at some point in the near future, so I'm particularly interested in being able to state that this functor is prorepresentable.

Christian Merten (Mar 24 2024 at 22:30):

By "this functor" you mean the functor sending a representation over kk to the set of lifts to RR?

Kevin Buzzard (Mar 24 2024 at 22:34):

Yes that's right, sorry for being unclear!

Kevin Buzzard (Mar 24 2024 at 22:36):

In fact the Mazur/Wiles situation has G a topological group and all representations continuous (i.e. with open kernel).

Kevin Buzzard (Mar 24 2024 at 22:38):

The idea is that there is a universal representation to GLn(Runiv)GL_n(R^{univ}) explaining all lifts but now RunivR^{univ} is a pro-object in the category of these finite rings, so it can be thought of as a profinite ring.

Christian Merten (Mar 24 2024 at 22:41):

Kevin Buzzard said:

Yes that's right, sorry for being unclear!

So everything covariant here, I take that as a vote for the FGA definition.

Christian Merten (Mar 24 2024 at 22:43):

Kevin Buzzard said:

In fact the Mazur/Wiles situation has G a topological group and all representations continuous (i.e. with open kernel).

This reminds me that I also need a proper definition of continuous representations for Galois categories (currently its very ad hoc).

Markus Himmel (Mar 25 2024 at 07:17):

I'm happy with any definition for the ind-category and the pro-category as long as there are equivalences IndCategory C ≌ FullSubcategory IsIndObject (where IsIndObject A might as well be defined as IsFiltered (CostructuredArrow yoneda A) ∧ FinallySmall.{v} (CostructuredArrow yoneda A)) and ProCategory C ≌ (IndCategory Cᵒᵖ)ᵒᵖ compatible with the various Yoneda embeddings and inclusions. I'm primarily interested in abstract limit-colimit properties of the categories and functors C ⥤ IndCategory C, IndCategory C ⥤ Cᵒᵖ ⥤ Type v, C ⥤ ProCategory C, ProCategory C ⥤ (C ⥤ Type v)ᵒᵖ, and everything I need follows from the two equivalences above. My only plan regarding the category of pro-objects so far was to transfer all the abstract properties from the category of ind-objects using the above equivalence. So I think that we should choose whatever definitions make working with ind-objects and pro-objects easiest in practice, and I should be able to make the formal stuff work form there.

Markus Himmel (Mar 25 2024 at 07:25):

Regarding the pro-yoneda lemma: I don't think something related is on my roadmap. I have a version of the Yoneda lemma involving colimits here, but it's different (the colimit is in the codomain instead of the domain).

Markus Himmel (Mar 25 2024 at 07:42):

To answer the more general question about my plans for ind-objects: I'm currently working on the following things:

  • ind-objects are closed under filtered colimits (this is done here, I'm currently in the process of PRing the prerequisites)
  • if C (is small and) has finite limits, then a presheaf is an ind-object if and only if it preserves finite limits
  • hom-sets between ind-objects are small
  • prerequisites about comma categories needed for the description of morphisms of ind-objects in terms of natural transformations of the functors defining them (after a suitable restriction)

There are many more things that I will definitely need:

  • the universal property
  • the functor C ⥤ IndCategory C preserves finite colimits
  • if C has finite limits, then IndCategory C has finite limits and the functors C ⥤ IndCategory C and IndCategory C ⥤ Cᵒᵖ ⥤ Type v preserve finite limits
  • if C has finite colimits, then IndCategory C has finite colimits (and hence also small colimits)

From there, my plan is to move on to the case where C is small and abelian, showing the equivalence between IndCategory C and LeftExactFunctor C AddCommGroup and working towards the statement that IndCategory C is a Grothendieck category.

Markus Himmel (Mar 25 2024 at 07:54):

One thing I've been wondering about is the characterization of hom-sets of pro-objects in terms of limits of colimits of hom-sets in C, see for example Lemma 2.6 on the nlab page on pro-objects. Kashiwara-Schapira only seem to need this to show that the pro-category is locally small. Is this characterization useful in applications? If so, it might be a good time to start thinking about how to make it ergonomic in Lean.

More generally, how do people work with morphisms of ind-objects and pro-objects in practice?

Kevin Buzzard (Mar 25 2024 at 07:54):

I am slightly nervous about the plan "prove everything for ind objects and deduce for pro objects" but only because in mathlib right now the general principle seems to be "do everything twice rather than attempting to deduce eg the theory of colimits from the theory of limits"

Kevin Buzzard (Mar 25 2024 at 07:58):

I think that in the FLT work people just informally pass from the pro-objects in the category of finite-as-a-type rings with residue field Z/p to an appropriate category of complete local Z_p-algebras with residue field Z/p and continuous morphisms...

Markus Himmel (Mar 25 2024 at 08:10):

Kevin Buzzard said:

I am slightly nervous about the plan "prove everything for ind objects and deduce for pro objects" but only because I'm mathlib right now the general principle seems to be "do everything twice rather than attempting to deduce eg the theory of colimits from the theory of limits"

My current vision for this is that everything is stated twice, but all the necessary infrastructure should be provided to transfer proofs, and longer proofs should not be duplicated. A simple example where this works is file#CategoryTheory/Filtered/Final. I think that we're in a much much better position for this than a few years ago, but there is still a lot of work to do. For example, file#CategoryTheory/Limits/Preserves/Opposites will need to grow by a factor of six to cover all necessary cases, and I'm currently thinking about how to make this happen while staying sane. Still, I think that this is a worthwhile approach that will increase productivity and usability in the long run.

Christian Merten (Mar 25 2024 at 08:35):

Kevin Buzzard said:

I think that in the FLT work people just informally pass from the pro-objects in the category of finite-as-a-type rings with residue field Z/p to an appropriate category of complete local Z_p-algebras with residue field Z/p and continuous morphisms...

Is the index category in the "lifts of representations" example naturally small? And maybe more importantly, if the lifts functor lands in Type v, is the indexing category naturally in Type v?
(The reason I am asking this: In my example, fibre functors of Galois categories, this does not happen, if one does not assume that the Galois category in question is itself small. This does not cause issues (yet), but prevents me from using the current ind-object (better: pro-object) setup (which is not a problem at all, since I don't need any categorical properties of ind/pro objects).

Kevin Buzzard (Mar 25 2024 at 08:37):

The finite rings are all in Type and the pro-objects are limits over types of finite objects (eg the p-adic integers is a limit over n in Nat of Z/p^n) so they're also in Type. Does this answer your question or is there more to it?

Christian Merten (Mar 25 2024 at 08:41):

If by the "pro-objects are limits over types" you mean the "pro-objects are limits indexed over elements of Type" then this answers my question and it should fit in the current setup.

Christian Merten (Mar 25 2024 at 08:50):

Markus Himmel said:

One thing I've been wondering about is the characterization of hom-sets of pro-objects in terms of limits of colimits of hom-sets in C, see for example Lemma 2.6 on the nlab page on pro-objects. Kashiwara-Schapira only seem to need this to show that the pro-category is locally small. Is this characterization useful in applications? If so, it might be a good time to start thinking about how to make it ergonomic in Lean.

More generally, how do people work with morphisms of ind-objects and pro-objects in practice?

I have ever only used the pro-yoneda lemmas, the one with colim on the left and the one with colim on the right, to speak about morphisms of pro objects (identifying the pro-object with the functor it represents). I think, since nlab defines pro objects to be the full subcategory of pro-representable functors, the characterisation in lemma 2.6 should follow from these.

Kyle Miller (Mar 25 2024 at 17:06):

In topology, one way pro-objects show up is filters. If you take the open neighborhood filter in a space XX at a point xx (call it FxF_x) and you let YY be a space standing for itself using the trivial filter, then hom(Fx,Y)\hom(F_x,Y) of topological/smooth/etc. pro-manifolds is the same thing as the set of germs of functions XYX\to Y centered at xx, which you can see from the lim/colim characterization. This is a special situation though, since (at least for smooth manifolds) you can use extension theorems to get a surjective map hom(X,Y)hom(Fx,Y)\hom(X,Y)\to\hom(F_x,Y) to represent every germ using some smooth map XYX\to Y.

For any open filters FF on XX and GG on YY, then the lim/colim characterization tells you how to make sense of hom(F,G)\hom(F,G). For every open neighborhood VV in GG there is an open neighborhood UU in FF and a morphism UVU\to V, and these all need to be compatible with respect to restrictions. (Interesting how that looks suspiciously like some sort of continuity condition when written this way.)

If you have a smooth map XYX\to Y that sends a closed subspace AA to a closed subspace BB, then you can "restrict" this be a smooth map "ABA\to B" in the pro-object sense, by replacing AA and BB with the filters of all open sets containing AA and BB. Such a pro-morphism contains the map ABA\to B itself, but it also contains the infinitesimal information about the map.

Adam Topaz (Apr 08 2024 at 20:38):

@Jack McKoen


Last updated: May 02 2025 at 03:31 UTC