Level.agda 414 B

1234567891011121314151617
  1. {-# OPTIONS --without-K #-}
  2. ------------------------------------------------------------------------
  3. -- Universe levels
  4. ------------------------------------------------------------------------
  5. module Common.Level where
  6. open import Agda.Primitive public using (Level; lzero; lsuc; _⊔_)
  7. -- Lifting.
  8. record Lift {a ℓ} (A : Set a) : Set (a ⊔ ℓ) where
  9. constructor lift
  10. field lower : A
  11. open Lift public