RTP.agda 979 B

12345678910111213141516171819202122232425262728293031323334353637383940414243
  1. module RTP where
  2. open import RTN public
  3. {-
  4. data Bool : Set where
  5. False : Bool
  6. True : Bool
  7. -}
  8. postulate
  9. Int : Set
  10. String : Set
  11. Float : Set
  12. Char : Set
  13. {-# BUILTIN FLOAT Float #-}
  14. {-# BUILTIN STRING String #-}
  15. -- postulate primShowBool : Bool -> String
  16. postulate primShowInt : Int -> String
  17. postulate primShowChar : Char -> String
  18. postulate primStringAppend : String -> String -> String
  19. postulate primStringReverse : String -> String
  20. -- postulate primStringToList : String -> List Char
  21. -- postulate primStringFromList
  22. -- Int stuff
  23. postulate primIntZero : Int
  24. postulate primIntOne : Int
  25. postulate primIntSucc : Int -> Int
  26. postulate primNatToInt : Nat -> Int
  27. postulate primIntToNat : Int -> Nat
  28. postulate primIntAdd : Int -> Int -> Int
  29. postulate primIntSub : Int -> Int -> Int
  30. postulate primIntMul : Int -> Int -> Int
  31. postulate primIntDiv : Int -> Int -> Int
  32. postulate primIntMod : Int -> Int -> Int