2018-02-16 11:03:02 +00:00
|
|
|
|
module Cat.Wishlist where
|
|
|
|
|
|
2018-02-19 10:25:16 +00:00
|
|
|
|
open import Level
|
2018-02-16 11:03:02 +00:00
|
|
|
|
open import Cubical.NType
|
|
|
|
|
open import Data.Nat using (_≤_ ; z≤n ; s≤s)
|
|
|
|
|
|
|
|
|
|
postulate ntypeCommulative : ∀ {ℓ n m} {A : Set ℓ} → n ≤ m → HasLevel ⟨ n ⟩₋₂ A → HasLevel ⟨ m ⟩₋₂ A
|
2018-02-19 10:25:16 +00:00
|
|
|
|
|
|
|
|
|
-- This follows from [HoTT-book: §7.1.10]
|
|
|
|
|
-- Andrea says the proof is in `cubical` but I can't find it.
|
|
|
|
|
postulate isSetIsProp : {ℓ : Level} → {A : Set ℓ} → isProp (isSet A)
|