view freyd.agda @ 304:bd7b3f3d1d4c

Freyd Adjoint Functor Theorem
author Shinji KONO <kono@ie.u-ryukyu.ac.jp>
date Sun, 05 Jan 2014 08:46:31 +0900
parents
children 211f6bec9b4a
line wrap: on
line source

open import Category -- https://github.com/konn/category-agda                                                                                     
open import Level
open import Category.Sets

module freyd {c₁ c₂ ℓ : Level} (A : Category c₁ c₂ ℓ) 
     (C : Category zero zero zero )
  where

open import Relation.Binary.Core

postulate ≈→≡ : {a b : Obj C } { x y : Hom C a b } →  (x≈y : C [ x ≈ y  ]) → x ≡ y


-- record SmallCategory