2014-10-09 05:57:41 +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
|
|
|
|
|
|
|
|
|
|
import .basic .constructions
|
|
|
|
|
|
|
|
|
|
open eq eq.ops category functor natural_transformation category.ops prod category.product
|
|
|
|
|
|
|
|
|
|
namespace adjoint
|
|
|
|
|
--representable functor
|
|
|
|
|
|
|
|
|
|
definition foo {obC : Type} (C : category obC) : C ×c C ⇒ C ×c C := functor.id
|
|
|
|
|
|
|
|
|
|
definition Hom {obC : Type} (C : category obC) : Cᵒᵖ ×c C ⇒ type :=
|
|
|
|
|
@functor.mk _ _ _ _ (λ a, hom (pr1 a) (pr2 a))
|
2014-10-09 06:44:09 +00:00
|
|
|
|
(λ a b f h, pr2 f ∘ h ∘ pr1 f)
|
|
|
|
|
(λ a, funext (λh, !id_left ⬝ !id_right))
|
|
|
|
|
(λ a b c g f, funext (λh,
|
2014-10-09 05:57:41 +00:00
|
|
|
|
show (pr2 g ∘ pr2 f) ∘ h ∘ (pr1 f ∘ pr1 g) = pr2 g ∘ (pr2 f ∘ h ∘ pr1 f) ∘ pr1 g, from sorry))
|
|
|
|
|
--I'm lazy, waiting for automation to fill this
|
|
|
|
|
|
2014-10-10 01:01:06 +00:00
|
|
|
|
variables {obC obD : Type} (C : category obC) {D : category obD}
|
2014-10-09 05:57:41 +00:00
|
|
|
|
|
2014-10-12 20:06:00 +00:00
|
|
|
|
variables (f : Cᵒᵖ ×c C ⇒ C ×c C) (g : C ×c C ⇒ C ×c C)
|
|
|
|
|
check g ∘f f
|
|
|
|
|
|
|
|
|
|
check natural_transformation (Hom D)
|
|
|
|
|
|
2014-10-09 07:05:37 +00:00
|
|
|
|
definition adjoint (F : C ⇒ D) (G : D ⇒ C) :=
|
|
|
|
|
natural_transformation (@functor.compose _ _ _ _ _ _ (Hom D) sorry)
|
2014-10-09 06:44:09 +00:00
|
|
|
|
--(Hom C ∘f sorry)
|
2014-10-09 07:05:37 +00:00
|
|
|
|
--product.prod_functor (opposite.opposite_functor F) (functor.ID D)
|
2014-10-09 05:57:41 +00:00
|
|
|
|
end adjoint
|