Zulip Chat Archive

Stream: maths

Topic: topology theorems for free via adjoint functors?


Kevin Buzzard (Dec 17 2024 at 00:07):

Over the last few months I've been developing a theory of the docs#moduleTopology , this is a canonical topology on a module over a topological ring. One abstract definition of it is as follows: if RR is a topological ring then a topological module MM for RR is an RR-module equipped with a topology such that +:M×MM+:M\times M\to M and :R×MM\bullet:R\times M\to M are both continuous. There's a forgetful functor FF from the category of topological RR-modules to the category of RR-modules, and this functor has an adjoint TT such that Hom(T(A),B)=Hom(A,F(B))Hom(T(A),B)=Hom(A,F(B)) (I always forget which way around these things are -- I think TT is a left adjoint?); this functor TT equips a module over a topological ring with its module topology (adjointness is basically docs#IsModuleTopology.continuous_of_linearMap ).

I'm about to launch into PRing proofs of statements such as: if two modules over a topological ring are both given the module topology, then the product topology has the module topology (and similar for finite products). But can I get such results for free from some adjoint functor nonsense argument?

Yaël Dillies (Dec 17 2024 at 06:31):

Product is a limit and right adjoints preserve limits. So F(A×B)=F(A)×F(B)F(A × B) = F(A) × F(B). If you want T(A×B)=T(A)×T(B)T(A × B) = T(A) × T(B) instead, then you need to find a left adjoint LL to TT, so that Hom(L(A),B)=Hom(A,T(B))\mathrm{Hom}(L(A), B) = \mathrm{Hom}(A, T(B))

Johan Commelin (Dec 17 2024 at 06:57):

Also, you will need to define the category of topological modules, and understand that what CategoryTheory thinks tje product should be, matches with what you want.

Kevin Buzzard (Dec 17 2024 at 07:53):

Product of modules is also a colimit so it sounds like I could do it this way? I didn't check the details though. The proof I have in FLT involves a big fight with the typeclass system so I was wondering whether this was a viable alternative. But in thinking how the category theory argument might look I realised that perhaps a type synonym in the middle of the non-category proof might save me.

Kevin Buzzard (Dec 17 2024 at 07:56):

I can't quite work out whether category theory not being useful here is something I should be annoyed about, or whether it's just showing my lack of understanding of all the details which would go into a category theory argument

Yaël Dillies (Dec 17 2024 at 08:40):

Kevin Buzzard said:

Product of modules is also a colimit

Good point, but the product of topological modules isn't a colimit, right?

Yaël Dillies (Dec 17 2024 at 08:43):

At least, the fact that the product of modules is a colimit is docs#LinearMap.coprodEquiv, and we don't have ContinuousLinearMap.coprodEquiv

Yaël Dillies (Dec 17 2024 at 11:04):

Okay well that was easy: #20016

Kevin Buzzard (Dec 17 2024 at 11:27):

Using a type synonym has solved my problems.

Yaël Dillies (Dec 17 2024 at 11:36):

For a topological RR-module MM, is there an easy way to construct a topological RR-module NN such that MHom(M,N)M ≅ \mathrm{Hom}(M, N)?

Yaël Dillies (Dec 17 2024 at 11:38):

If so, you can chain this with coprodEquiv and get T(A×B)=T(A)×T(B)T(A × B) = T(A) × T(B)

Kevin Buzzard (Dec 17 2024 at 11:55):

Yaël Dillies said:

For a topological RR-module MM, is there an easy way to construct a topological RR-module NN such that MHom(M,N)M ≅ \mathrm{Hom}(M, N)?

No that doesn't look right. Even without the topology this doesn't look right.

Yaël Dillies (Dec 17 2024 at 12:04):

So coyoneda doesn't hold for Mod\mathrm{Mod}?

Kevin Buzzard (Dec 17 2024 at 12:19):

M=Hom_R(R,M) but you can't have something the other way around, if that's what you're asking.

Kevin Buzzard (Dec 17 2024 at 12:20):

Hom_R(M,N) for a fixed N is contravariant in M so you can't expect it to be related to M or even have a map to or from M in general. (but I don't know what "coyoneda doesn't hold for Mod" means)

Yaël Dillies (Dec 17 2024 at 12:29):

What I am saying is that I can prove Hom(T(A×B),C)Hom(T(A)×T(B),C)\mathrm{Hom}(T(A \times B), C) \cong \mathrm{Hom}(T(A) \times T(B), C) for all CC, but I don't know how to get T(A×B)T(A)×T(B)T(A \times B) \cong T(A) \times T(B) from it. Unless I have misunderstood, the way to get this is the Yoneda lemma.

Yaël Dillies (Dec 17 2024 at 12:31):

Oh, is the idea that I set C:=T(A×B)C := T(A × B) and push forward the identity morphism, then set C:=T(A)×T(B)C := T(A) × T(B) and pull back the identity morphism?

Kevin Buzzard (Dec 17 2024 at 12:37):

Just to be clear, I've now done this in a category-free way in FLT having found a way to avoid the typeclass battle (set P:= M x N with module topology, and let Lean believe that M x N has product topology)

Adam Topaz (Dec 17 2024 at 12:41):

I don't see how tricks with yoneda will help here. Constructing an isomoprhism between T(A×B)T(A \times B) and T(A)×T(B)T(A) \times T(B) is equivalent to constructing a natural isomorphism after applying the coyoneda embedding. There is a natural morphism T(A×B)T(A)×T(B)T(A \times B) \to T(A) \times T(B) and presumably it would be easier to prove that this is an isomoprhism.

Kevin Buzzard (Dec 17 2024 at 13:00):

FWIW my non-category proof had some content. The key argument was proving that the identity map from (M x N, product topology) to (M x N, module topology) was continuous, which involved writing it as the function sending mn to i1(pr1(mn))+i2(pr2(mn)) where the pr's are projections from products hence continuous, the i's are inclusions M -> P (P:=MxN with module topology) are linear and hence continuous, and addition on P is continuous.

Adam Topaz (Dec 17 2024 at 13:01):

Note that the topology on T(A)T(A) is sInf ..., and the topology on the product is ... \sqcap .... The map T(A×B)T(A)×T(B)T(A \times B) \to T(A) \times T(B) is the identity on the underlying modules, so it suffices to show that the topologies agree, and so it looks like this could be accomplished using the fact that sInf commutes with \sqcap in a suitable lattice.

Kevin Buzzard (Dec 17 2024 at 13:01):

This (the fact that my argument had some content) was another reason why I was interested about whether it could all be done with abstract nonsense (but not interested enough to think about it myself)

Adam Topaz (Dec 17 2024 at 13:04):

In fact your definition of T(M)T(M) is as a limit over the diagram of all topological module structures on this fixed MM. And since limits commute with limits, this could be a abstract-nonsense approach.

Mitchell Lee (Dec 17 2024 at 13:04):

It is enough to show that the direct sum of two topological RR-modules MM and NN, in the category of topological RR-modules, is the usual direct sum MNM \oplus N with the product topology. Then TT is a left adjoint, so it is right exact, so it preserves direct sums.

Mitchell Lee (Dec 17 2024 at 13:04):

However, it is not obvious to me whether this fact can be proved with abstract nonsense.

Mitchell Lee (Dec 17 2024 at 13:13):

There is also this proposition which makes it easier to prove that something is a direct sum, but I think there is still something to be done: https://ncatlab.org/nlab/show/additive+category#ProductsAreBiproducts

Mitchell Lee (Dec 17 2024 at 13:25):

This would also imply thay the category of topological RR-modules is an additive category, which might be useful for other purposes.

Mitchell Lee (Dec 17 2024 at 18:10):

Ok, I found a lemma in mathlib that lets you do all this:

https://leanprover-community.github.io/mathlib4_docs/Mathlib/CategoryTheory/Preadditive/Biproducts.html#CategoryTheory.Limits.isBinaryBilimitOfTotal

Mitchell Lee (Dec 17 2024 at 18:17):

This can be used to prove that the direct sum (binary biproduct) of MM and NN in the category of topological RR-modules is the Cartesian product M×NM \times N with the product topology. It might still just be easier to prove your theorems directly without category theory, though.

Kevin Buzzard (Dec 17 2024 at 19:18):

Mitchell Lee said:

It might still just be easier to prove your theorems directly without category theory, though.

https://github.com/ImperialCollegeLondon/FLT/blob/8a133980a700b1a25a465f08c2dec56e367ccd78/FLT/Mathlib/Topology/Algebra/Module/ModuleTopology.lean#L188-L221

Mitchell Lee (Dec 17 2024 at 19:29):

Yeah, that does look easier

Kevin Buzzard (Dec 17 2024 at 19:43):

FWIW here's what that proof looked like 2 days ago, and this was what inspired the question. I then had the idea of using a type synonym and all my problems evaporated.


Last updated: May 02 2025 at 03:31 UTC