Erased-cubical-FFI.agda 321 B

1234567891011121314
  1. {-# OPTIONS --erased-cubical --no-main --save-metas #-}
  2. open import Agda.Builtin.Bool
  3. open import Erased-cubical-Cubical
  4. postulate
  5. f : Not-compiled → Bool
  6. -- It is at the time of writing not possible to give a COMPILE GHC
  7. -- pragma for f, because Not-compiled is not compiled.
  8. {-# COMPILE GHC f = \_ -> True #-}