src/HOL/Hoare/HoareAbort.thy
changeset 30510 4120fc59dd85
parent 30304 d8e4cd2ac2a1
child 30549 d2d7874648bd
--- a/src/HOL/Hoare/HoareAbort.thy	Fri Mar 13 19:53:09 2009 +0100
+++ b/src/HOL/Hoare/HoareAbort.thy	Fri Mar 13 19:58:26 2009 +0100
@@ -246,12 +246,12 @@
 use "hoare_tac.ML"
 
 method_setup vcg = {*
-  Method.ctxt_args (fn ctxt => Method.SIMPLE_METHOD' (hoare_tac ctxt (K all_tac))) *}
+  Method.ctxt_args (fn ctxt => SIMPLE_METHOD' (hoare_tac ctxt (K all_tac))) *}
   "verification condition generator"
 
 method_setup vcg_simp = {*
   Method.ctxt_args (fn ctxt =>
-    Method.SIMPLE_METHOD' (hoare_tac ctxt (asm_full_simp_tac (local_simpset_of ctxt)))) *}
+    SIMPLE_METHOD' (hoare_tac ctxt (asm_full_simp_tac (local_simpset_of ctxt)))) *}
   "verification condition generator plus simplification"
 
 (* Special syntax for guarded statements and guarded array updates: *)