diff -r fe9d746b273e -r bf2fecda8383 src/Tools/Haskell/Build.thy --- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/Tools/Haskell/Build.thy Sat Nov 03 19:33:15 2018 +0100 @@ -0,0 +1,24 @@ +(* Title: Tools/Haskell/Build.thy + Author: Makarius +*) + +section \Build Isabelle/Haskell modules\ + +theory Build imports Haskell +begin + +ML_command \ + Isabelle_System.with_tmp_dir "ghc" (fn dir => + let + val (out, rc) = + Isabelle_System.bash_output + (cat_lines + ["set -e", + "cd " ^ File.bash_path dir, + "cp " ^ File.bash_paths Haskell.source_modules ^ " .", + "\"$ISABELLE_GHC\" " ^ File.bash_paths (map Path.base Haskell.source_modules)]); + in if rc = 0 then writeln out else error out end + ) +\ + +end