discontinued futile attempt to hardwire build options into the image, sequential mode is enabled more robustly at runtime (cf. 3b0a60eee56e);
authorwenzelm
Mon, 24 Sep 2012 16:13:56 +0200
changeset 49550 0a82e98fd4a3
parent 49549 3b0a60eee56e
child 49551 9b12fcd0a889
discontinued futile attempt to hardwire build options into the image, sequential mode is enabled more robustly at runtime (cf. 3b0a60eee56e);
src/HOL/Mirabelle/Mirabelle.thy
--- a/src/HOL/Mirabelle/Mirabelle.thy	Mon Sep 24 15:37:58 2012 +0200
+++ b/src/HOL/Mirabelle/Mirabelle.thy	Mon Sep 24 16:13:56 2012 +0200
@@ -9,10 +9,6 @@
 ML_file "Tools/mirabelle.ML"
 ML_file "../TPTP/sledgehammer_tactics.ML"
 
-(* no multithreading, no parallel proofs *)  (* FIXME *)
-ML {* Multithreading.max_threads := 1 *}
-ML {* Goal.parallel_proofs := 0 *}
-
 ML {* Toplevel.add_hook Mirabelle.step_hook *}
 
 ML {*