src/HOL/UNITY/UNITY_Main.thy
changeset 30549 d2d7874648bd
parent 30510 4120fc59dd85
child 32149 ef59550a55d3
--- a/src/HOL/UNITY/UNITY_Main.thy	Mon Mar 16 17:51:24 2009 +0100
+++ b/src/HOL/UNITY/UNITY_Main.thy	Mon Mar 16 18:24:30 2009 +0100
@@ -10,15 +10,13 @@
 uses "UNITY_tactics.ML" begin
 
 method_setup safety = {*
-    Method.ctxt_args (fn ctxt =>
+    Scan.succeed (fn ctxt =>
         SIMPLE_METHOD' (constrains_tac (local_clasimpset_of ctxt))) *}
     "for proving safety properties"
 
 method_setup ensures_tac = {*
-    fn args => fn ctxt =>
-        Method.goal_args' (Scan.lift Args.name_source)
-           (ensures_tac (local_clasimpset_of ctxt))
-           args ctxt *}
-    "for proving progress properties"
+  Args.goal_spec -- Scan.lift Args.name_source >>
+  (fn (quant, s) => fn ctxt => SIMPLE_METHOD'' quant (ensures_tac (local_clasimpset_of ctxt) s))
+*} "for proving progress properties"
 
 end