Zulip Chat Archive
Stream: Is there code for X?
Topic: flip eq curry swap uncurry
Adam Topaz (Dec 30 2021 at 18:01):
I would be surprised if the following doesn't already exist, but I couldn't find it.
import category_theory.currying
open category_theory
variables {C D E : Type*} [category C] [category D] [category E]
example (F : C ⥤ D ⥤ E) :
F.flip ≅ curry.obj (category_theory.prod.swap _ _ ⋙ uncurry.obj F) :=
nat_iso.of_components (λ d, nat_iso.of_components (λ c, eq_to_iso rfl) $ by tidy) $ by tidy
Adam Topaz (Dec 30 2021 at 18:08):
Last updated: Dec 20 2023 at 11:08 UTC