cat/src/Cat/Wishlist.agda

17 lines
518 B
Agda
Raw Normal View History

module Cat.Wishlist where
2018-02-19 10:25:16 +00:00
open import Level
open import Cubical.NType
open import Data.Nat using (_≤_ ; z≤n ; s≤s)
open import Cubical.NType.Properties public using (propHasLevel)
postulate ntypeCommulative : { n m} {A : Set } n m HasLevel n ⟩₋₂ A HasLevel m ⟩₋₂ A
2018-02-19 10:25:16 +00:00
module _ { : Level} {A : Set } where
isSetIsProp : isProp (isSet A)
isSetIsProp = propHasLevel (S (S ⟨-2⟩))
propIsProp : isProp (isProp A)
propIsProp = propHasLevel (S ⟨-2⟩)