ImportB.agda 354 B

1234567891011121314
  1. module Issue2486.ImportB where
  2. open import Issue2486.Haskell
  3. {-# FOREIGN GHC data BBool = BTrue | BFalse #-}
  4. data BBool : Set where
  5. BTrue BFalse : BBool
  6. {-# COMPILE GHC BBool = data BBool ( BTrue | BFalse ) #-}
  7. postulate BList : Set → Set
  8. {-# FOREIGN GHC import MAlonzo.Code.Issue2486.Haskell (MyList) #-}
  9. {-# COMPILE GHC BList = type MyList #-}