discontinued futile attempt to hardwire build options into the image, sequential mode is enabled more robustly at runtime (cf. 3b0a60eee56e);
--- 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 {*