Size.agda 321 B

1234567891011
  1. {-# OPTIONS --without-K --sized-types #-}
  2. ------------------------------------------------------------------------
  3. -- From the Agda standard library
  4. --
  5. -- Sizes for Agda's sized types
  6. ------------------------------------------------------------------------
  7. module Common.Size where
  8. open import Agda.Builtin.Size public