delect installed ATPs dynamically, _not_ at image built time
authorblanchet
Fri, 14 May 2010 11:20:09 +0200
changeset 36908 fb18db78be80
parent 36907 9063a5b2b2bb
child 36909 7d5587f6d5f7
delect installed ATPs dynamically, _not_ at image built time
src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Thu May 13 15:09:42 2010 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML	Fri May 14 11:20:09 2010 +0200
@@ -64,7 +64,7 @@
 
 (*** parameters ***)
 
-val atps = Unsynchronized.ref (default_atps_param_value ())
+val atps = Unsynchronized.ref ""
 val timeout = Unsynchronized.ref 60
 val full_types = Unsynchronized.ref false
 
@@ -112,7 +112,7 @@
    ("ignore_no_atp", "respect_no_atp"),
    ("theory_irrelevant", "theory_relevant"),
    ("dont_follow_defs", "follow_defs"),
-   ("metis_proof", "isar_proof")]
+   ("no_isar_proof", "isar_proof")]
 
 val params_for_minimize =
   ["debug", "verbose", "overlord", "full_types", "explicit_apply",
@@ -152,7 +152,7 @@
 fun default_raw_params thy =
   Data.get thy
   |> fold (AList.default (op =))
-          [("atps", [!atps]),
+          [("atps", [case !atps of "" => default_atps_param_value () | s => s]),
            ("full_types", [if !full_types then "true" else "false"]),
            ("timeout", let val timeout = !timeout in
                          [if timeout <= 0 then "none"