cat/src/Cat/Category/Properties.agda

24 lines
577 B
Agda
Raw Normal View History

{-# OPTIONS --allow-unsolved-metas #-}
module Cat.Category.Properties where
open import Cat.Category
open import Cat.Functor
open import Cat.Categories.Sets
module _ {a a' b b'} where
Exponential : Category {a} {a'} Category {b} {b'} Category {{!!}} {{!!}}
Exponential A B = record
{ Object = {!!}
; Arrow = {!!}
; 𝟙 = {!!}
; _⊕_ = {!!}
; assoc = {!!}
; ident = {!!}
}
_⇑_ = Exponential
yoneda : { '} { : Category {} {'}} Functor (Sets (Opposite ))
yoneda = {!!}