diff --git a/thys/Buchi_Complementation/Complementation_Build.thy b/thys/Buchi_Complementation/Complementation_Build.thy --- a/thys/Buchi_Complementation/Complementation_Build.thy +++ b/thys/Buchi_Complementation/Complementation_Build.thy @@ -1,27 +1,27 @@ section \Build and test exported program with MLton\ theory Complementation_Build imports Complementation_Final begin external_file \code/Autool.mlb\ external_file \code/Prelude.sml\ external_file \code/Autool.sml\ compile_generated_files \<^marker>\contributor Makarius\ \code/Complementation.ML\ (in Complementation_Final) external_files \code/Autool.mlb\ \code/Prelude.sml\ \code/Autool.sml\ export_files \code/Complementation.sml\ and \code/Autool\ (exe) where \fn dir => let val exec = Generated_Files.execute (dir + Path.basic "code"); val _ = exec \Prepare\ "mv Complementation.ML Complementation.sml"; - val _ = exec \Compilation\ (File.bash_path \<^path>\$ISABELLE_MLTON\ ^ + val _ = exec \Compilation\ (\<^verbatim>\"$ISABELLE_MLTON" $ISABELLE_MLTON_OPTIONS \ ^ " -profile time -default-type intinf Autool.mlb"); val _ = exec \Test\ "./Autool help"; in () end\ end \ No newline at end of file diff --git a/thys/PAC_Checker/PAC_Checker_MLton.thy b/thys/PAC_Checker/PAC_Checker_MLton.thy --- a/thys/PAC_Checker/PAC_Checker_MLton.thy +++ b/thys/PAC_Checker/PAC_Checker_MLton.thy @@ -1,34 +1,34 @@ (* File: PAC_Checker_MLton.thy Author: Mathias Fleury, Daniela Kaufmann, JKU Maintainer: Mathias Fleury, JKU *) theory PAC_Checker_MLton imports PAC_Checker_Synthesis begin export_code PAC_checker_l_impl PAC_update_impl PAC_empty_impl the_error is_cfailed is_cfound int_of_integer Del Add Mult nat_of_integer String.implode remap_polys_l_impl fully_normalize_poly_impl union_vars_poly_impl empty_vars_impl full_checker_l_impl check_step_impl CSUCCESS Extension hashcode_literal' version in SML_imp module_name PAC_Checker file_prefix "checker" text \Here is how to compile it:\ compile_generated_files _ external_files \code/parser.sml\ \code/pasteque.sml\ \code/pasteque.mlb\ where \fn dir => let val exec = Generated_Files.execute (dir + Path.basic "code"); val _ = exec \Compilation\ - (File.bash_path \<^path>\$ISABELLE_MLTON\ ^ " " ^ + (\<^verbatim>\"$ISABELLE_MLTON" $ISABELLE_MLTON_OPTIONS \ ^ "-const 'MLton.safe false' -verbose 1 -default-type int64 -output pasteque " ^ "-codegen native -inline 700 -cc-opt -O3 pasteque.mlb"); in () end\ end \ No newline at end of file