Erased-cubical-Cubical.agda 259 B

123456789101112
  1. {-# OPTIONS --cubical --save-metas #-}
  2. -- The code in this module should not be compiled. However, the
  3. -- following re-exported code should be compiled.
  4. open import Agda.Builtin.Bool public
  5. postulate
  6. easy : {A : Set} → A
  7. data Not-compiled : Set where