ExportAndUse.agda 241 B

12345678910111213141516
  1. module ExportAndUse where
  2. data Bool : Set where
  3. true false : Bool
  4. {-# COMPILE GHC Bool = data Bool (True | False) #-}
  5. foo : Bool → Bool
  6. foo true = false
  7. foo false = true
  8. {-# COMPILE GHC foo as foohs #-}
  9. test : Bool
  10. test = foo true