src/Provers/blast.ML
changeset 69593 3dda49e08b9d
parent 63280 d2d26ff708d7
child 79171 377260b2824d
--- a/src/Provers/blast.ML	Fri Jan 04 21:49:06 2019 +0100
+++ b/src/Provers/blast.ML	Fri Jan 04 23:22:53 2019 +0100
@@ -76,9 +76,9 @@
 
 (* options *)
 
-val depth_limit = Attrib.setup_config_int @{binding blast_depth_limit} (K 20);
-val (trace, _) = Attrib.config_bool @{binding blast_trace} (K false);
-val (stats, _) = Attrib.config_bool @{binding blast_stats} (K false);
+val depth_limit = Attrib.setup_config_int \<^binding>\<open>blast_depth_limit\<close> (K 20);
+val (trace, _) = Attrib.config_bool \<^binding>\<open>blast_trace\<close> (K false);
+val (stats, _) = Attrib.config_bool \<^binding>\<open>blast_stats\<close> (K false);
 
 
 datatype term =
@@ -418,12 +418,12 @@
 
 
 (* A1==>...An==>B  goes to  [A1,...,An], where B is not an implication *)
-fun strip_imp_prems (Const (@{const_name Pure.imp}, _) $ A $ B) =
+fun strip_imp_prems (Const (\<^const_name>\<open>Pure.imp\<close>, _) $ A $ B) =
       strip_Trueprop A :: strip_imp_prems B
   | strip_imp_prems _ = [];
 
 (* A1==>...An==>B  goes to B, where B is not an implication *)
-fun strip_imp_concl (Const (@{const_name Pure.imp}, _) $ A $ B) = strip_imp_concl B
+fun strip_imp_concl (Const (\<^const_name>\<open>Pure.imp\<close>, _) $ A $ B) = strip_imp_concl B
   | strip_imp_concl A = strip_Trueprop A;
 
 
@@ -443,7 +443,7 @@
           else P :: delete_concl Ps
       | _ => P :: delete_concl Ps);
 
-fun skoPrem state vars (Const (@{const_name Pure.all}, _) $ Abs (_, P)) =
+fun skoPrem state vars (Const (\<^const_name>\<open>Pure.all\<close>, _) $ Abs (_, P)) =
         skoPrem state vars (subst_bound (Skolem (gensym state "S", vars), P))
   | skoPrem _ _ P = P;
 
@@ -1188,7 +1188,7 @@
 (*Make a list of all the parameters in a subgoal, even if nested*)
 local open Term
 in
-fun discard_foralls (Const(@{const_name Pure.all},_)$Abs(a,T,t)) = discard_foralls t
+fun discard_foralls (Const(\<^const_name>\<open>Pure.all\<close>,_)$Abs(a,T,t)) = discard_foralls t
   | discard_foralls t = t;
 end;
 
@@ -1311,7 +1311,7 @@
 
 val _ =
   Theory.setup
-    (Method.setup @{binding blast}
+    (Method.setup \<^binding>\<open>blast\<close>
       (Scan.lift (Scan.option Parse.nat) --| Method.sections Classical.cla_modifiers >>
         (fn NONE => SIMPLE_METHOD' o blast_tac
           | SOME lim => (fn ctxt => SIMPLE_METHOD' (depth_tac ctxt lim))))