Zulip Chat Archive
Stream: mathlib4
Topic: Variation of `Functor.sum`
Sina Hazratpour 𓃵 (Apr 11 2024 at 19:23):
Functor.sum
defines a functor of type Sum A C ⥤ Sum B D
. I need a variation which has the type Sum A B ⥤ C
but I could not find it in CategoryTheory/Sums
.
Actually, if we define
def sum₂ (F : A ⥤ C) (G : B ⥤ C) : Sum A B ⥤ C where
then we have that sum F G = sumâ‚‚ (F â‹™ Sum.inl_) (G â‹™ Sum.inr_)
.
So it seems to me that sumâ‚‚
is a bit more fundamental than sum
the way it is defined.
Is it a good idea to add sumâ‚‚
to mathlib?
Adam Topaz (Apr 11 2024 at 19:27):
Are we really missing the (2-)universal property of docs#Sum ?
Sina Hazratpour 𓃵 (Apr 11 2024 at 19:29):
I was not pursuing that path, since i thought I might get into problem with the universes (aka size issue). Are you suggesting defining sumâ‚‚
as a gap map out of the sum in the large 2-category of (small) categories?
I'll try this.
Sina Hazratpour 𓃵 (Apr 11 2024 at 19:59):
@Adam Topaz
I think the situation is dual to docs#CategoryTheory.Functor.prod', might be a good idea to define Functor.sum'
?
Last updated: May 02 2025 at 03:31 UTC