[Agda] Compiling HelloWorld
Philippe de Rochambeau
phiroc at free.fr
Wed Apr 15 20:12:04 CEST 2020
Hello,
compiling the following code from the 2.6.1 Agda Documentation causes the below error message.
module HelloWorld where
open import Agda.Builtin.IO
open import Agda.Builtin.Unit
open import Agda.Builtin.String
postulate
putStrLn : String → IO ⊤
{-# FOREIGN GHC import qualified Data.Text.IO as Text #-}
{-# COMPILE GHC putStrLn = Text.putStrLn #-}
main : IO ⊤
main = putStrLn "Hello, World!"
Compilation error:
MAlonzo/RTE.hs:9:1: error:
Could not find module ‘Numeric.IEEE’
Use -v (or `:set -v` in ghci) to see a list of the files searched for.
|
9 | import Numeric.IEEE ( IEEE(identicalIEEE, nan) )
| ^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^^
How do you fix it?
Many thanks.
Philippe
-------------- next part --------------
An HTML attachment was scrubbed...
URL: <http://lists.chalmers.se/pipermail/agda/attachments/20200415/de1453a1/attachment.html>
More information about the Agda
mailing list