2014-12-22 15:33:29 -05:00
|
|
|
|
/-
|
|
|
|
|
Copyright (c) 2014 Floris van Doorn. All rights reserved.
|
|
|
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
|
|
|
|
|
|
Module: algebra.category.adjoint
|
|
|
|
|
Author: Floris van Doorn
|
|
|
|
|
-/
|
2014-10-09 01:57:41 -04:00
|
|
|
|
|
2014-11-03 19:22:30 -05:00
|
|
|
|
import .constructions
|
2014-10-09 01:57:41 -04:00
|
|
|
|
|
|
|
|
|
open eq eq.ops category functor natural_transformation category.ops prod category.product
|
|
|
|
|
|
|
|
|
|
namespace adjoint
|
|
|
|
|
|
2014-11-03 19:22:30 -05:00
|
|
|
|
-- definition Hom (C : Category) : Cᵒᵖ ×c C ⇒ type :=
|
|
|
|
|
-- functor.mk (λ a, hom (pr1 a) (pr2 a))
|
2014-11-24 20:24:30 -05:00
|
|
|
|
-- (λ a b f h, sorry)
|
|
|
|
|
-- (λ a, sorry)
|
|
|
|
|
-- (λ a b c g f, sorry)
|
2014-10-12 13:06:00 -07:00
|
|
|
|
|
2014-10-09 01:57:41 -04:00
|
|
|
|
end adjoint
|