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