src/Tools/Haskell/Test.thy
author wenzelm
Sat, 01 Dec 2018 16:11:59 +0100
changeset 69383 747f8b052e59
parent 69381 4c9b4e2c5460
child 69385 be9f187dcd50
permissions -rw-r--r--
clarified modules;

(*  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 \<^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