cat/src/Cat/CartesianClosed.agda

13 lines
331 B
Agda
Raw Normal View History

module Cat.CartesianClosed where
open import Agda.Primitive
open import Cat.Category
open import Cat.Product
open import Cat.Exponential
record CartesianClosed { ' : Level} ( : Category ') : Set ( ') where
field
{{hasProducts}} : HasProducts
{{hasExponentials}} : HasExponentials