src/HOL/Hoare/HoareAbort.thy
changeset 30549 d2d7874648bd
parent 30510 4120fc59dd85
child 32134 ee143615019c
--- a/src/HOL/Hoare/HoareAbort.thy	Mon Mar 16 17:51:24 2009 +0100
+++ b/src/HOL/Hoare/HoareAbort.thy	Mon Mar 16 18:24:30 2009 +0100
@@ -246,11 +246,11 @@
 use "hoare_tac.ML"
 
 method_setup vcg = {*
-  Method.ctxt_args (fn ctxt => SIMPLE_METHOD' (hoare_tac ctxt (K all_tac))) *}
+  Scan.succeed (fn ctxt => SIMPLE_METHOD' (hoare_tac ctxt (K all_tac))) *}
   "verification condition generator"
 
 method_setup vcg_simp = {*
-  Method.ctxt_args (fn ctxt =>
+  Scan.succeed (fn ctxt =>
     SIMPLE_METHOD' (hoare_tac ctxt (asm_full_simp_tac (local_simpset_of ctxt)))) *}
   "verification condition generator plus simplification"