Zulip Chat Archive

Stream: new members

Topic: Unique morphism between producs


Yakov Pechersky (Aug 06 2023 at 17:35):

I am trying to learn the category theory library in mathlib, and am having difficulty understanding how to tackle the following exercise using mathlib. I have a proof using my own home-brewed category definitions.
image.png

lemma AProd.lift_square_aux {G H : C} (φ : G  H) :
    Nonempty (Unique ({fg : G ×_C G  H ×_C H // fg  fstHom = fstHom  φ  fg  sndHom = sndHom  φ})) := by
  refine' ⟨⟨lift (fstHom  φ) (sndHom  φ), lift_comp_fst _ _, lift_comp_snd _ _⟩, _
  intro h, hl, hr
  exact Subtype.ext (lift_unique h hl hr)

Yakov Pechersky (Aug 06 2023 at 17:36):

The full code to make my proof work is here:

Full code

Yakov Pechersky (Aug 06 2023 at 17:37):

Where can I find some documentation/guide to understand how to reinterpret my proof in mathlib-style category theory defns?

Adam Topaz (Aug 06 2023 at 18:53):

This is a really poorly stated exercise imo.

Adam Topaz (Aug 06 2023 at 18:55):

It’s not true that there is a unique morphism. What is true is that there is a unique morphism such that the composition with the projections satisfies some commutative square involving phi.

Adam Topaz (Aug 06 2023 at 18:56):

That last point is left very implicit in the notation (ϕ,ϕ)(\phi,\phi).

Yakov Pechersky (Aug 06 2023 at 19:10):

Agreed. That's why I constrained the uniqueness to the subtype of homs such that composition equals composition with with phi.

Yakov Pechersky (Aug 06 2023 at 19:11):

Initially, I was stuck for a while because I didn't have that constraint. But then I realized that if there was another hom psi between G and H, that would induce another hom between the products.

Adam Topaz (Aug 06 2023 at 19:49):

The main definition you want to look at from mathlib would be docs#CategoryTheory.prod and the relevant api

Adam Topaz (Aug 06 2023 at 19:50):

we have docs#CategoryTheory.Limits.prod.map


Last updated: Dec 20 2023 at 11:08 UTC