cat/src/Cat/Category/CartesianClosed.agda

13 lines
358 B
Agda
Raw Normal View History

2018-02-05 13:59:53 +00:00
module Cat.Category.CartesianClosed where
open import Agda.Primitive
open import Cat.Category
2018-02-05 13:59:53 +00:00
open import Cat.Category.Product
open import Cat.Category.Exponential
record CartesianClosed { ' : Level} ( : Category ') : Set ( ') where
field
{{hasProducts}} : HasProducts
{{hasExponentials}} : HasExponentials