Frederik Hanghøj Iversen
7dc7a5aee3
Also adds a new module `Cat.Wishlist` of things I hope to put get from upstream `cubical`.
7 lines
236 B
Agda
7 lines
236 B
Agda
module Cat.Wishlist where
|
||
|
||
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
|