2018-02-05 13:59:53 +00:00
|
|
|
|
module Cat.Category.CartesianClosed where
|
2018-02-05 13:08:30 +00:00
|
|
|
|
|
|
|
|
|
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
|
2018-02-05 13:08:30 +00:00
|
|
|
|
|
|
|
|
|
record CartesianClosed {ℓ ℓ' : Level} (ℂ : Category ℓ ℓ') : Set (ℓ ⊔ ℓ') where
|
|
|
|
|
field
|
|
|
|
|
{{hasProducts}} : HasProducts ℂ
|
|
|
|
|
{{hasExponentials}} : HasExponentials ℂ
|