Zulip Chat Archive

Stream: Is there code for X?

Topic: product of two representable functors


Kevin Buzzard (Jan 20 2025 at 16:57):

Presumably under mild assumptions, the product of two representable functors is representable (by the product of the representing objects) and probably there are more general statements, such as finite limits of representable functors are representable. Or maybe I mean corepresentable, I am always confused by the ops here. But my question is whether we have the actual correct versions of these theorems? Presumably they are not too hard?

Joël Riou (Jan 20 2025 at 17:25):

I do not think we have these exact statements. We have some related material though:

  • The RepresentableBy/IsRepresentable API in the file CategoryTheory.Yoneda
  • yoneda_preservesLimit in CategoryTheory.Limits.Yoneda

Then, if you show that a diagram of representable functors is isomorphic to a composition F ⋙ yoneda, the result should follow.

(In order to even state what you want, you may also use the ClosedUnderLimitsOfShape API from CategoryTheory.Limits.FullSubcategory. Alternatively, if you would like to focus on the binary product case, it would be very reasonable to state and prove things very directly in terms of the RepresentableBy API.)

Adam Topaz (Jan 20 2025 at 20:23):

exact?% finds the following:

import Mathlib

open CategoryTheory Limits

example {C : Type*} [Category C] [HasLimits C] (X Y : C) :
   yoneda.obj (X  Y)  yoneda.obj X  yoneda.obj Y :=
  PreservesLimitPair.iso yoneda X Y

Last updated: May 02 2025 at 03:31 UTC