MAlonzo.agda 493 B

12345678910111213141516171819202122
  1. {-# OPTIONS --guardedness #-}
  2. module Common.MAlonzo where
  3. open import Common.Prelude hiding (putStrLn)
  4. open import Common.Coinduction
  5. {-# FOREIGN GHC import qualified Data.Text.IO #-}
  6. postulate
  7. putStrLn : ∞ String → IO Unit
  8. {-# COMPILE GHC putStrLn = Data.Text.IO.putStrLn . MAlonzo.RTE.flat #-}
  9. main = putStrLn (♯ "This is a dummy main routine.")
  10. mainPrint : String → _
  11. mainPrint s = putStrLn (♯ s)
  12. mainPrintNat : Nat → _
  13. mainPrintNat n = putStrLn (♯ (natToString n))