| author | wenzelm |
| Sun, 09 Dec 2018 20:19:31 +0100 | |
| changeset 69439 | 22d4cb91ea6d |
| parent 69385 | be9f187dcd50 |
| child 69444 | c3c9440cbf9b |
| permissions | -rw-r--r-- |
(* Title: Tools/Haskell/Test.thy Author: Makarius *) section \<open>Test build of Isabelle/Haskell modules\<close> theory Test imports Haskell begin ML \<open> Isabelle_System.with_tmp_dir "ghc" (fn dir => let val files = Generated_Files.write_files \<^theory>\<open>Haskell\<close> dir; val (out, rc) = Isabelle_System.bash_output (cat_lines ["set -e", "cd " ^ File.bash_path dir, "\"$ISABELLE_GHC\" " ^ File.bash_paths files]); in if rc = 0 then writeln out else error out end) \<close> end