src/HOL/Hoare/Hoare.thy
changeset 28457 25669513fd4c
parent 24472 943ef707396c
child 30304 d8e4cd2ac2a1
--- a/src/HOL/Hoare/Hoare.thy	Thu Oct 02 13:07:33 2008 +0200
+++ b/src/HOL/Hoare/Hoare.thy	Thu Oct 02 14:22:36 2008 +0200
@@ -9,7 +9,8 @@
 later.
 *)
 
-theory Hoare  imports Main
+theory Hoare
+imports Main
 uses ("hoare_tac.ML")
 begin
 
@@ -229,15 +230,16 @@
 lemma Compl_Collect: "-(Collect b) = {x. ~(b x)}"
   by blast
 
+lemmas AbortRule = SkipRule  -- "dummy version"
 use "hoare_tac.ML"
 
 method_setup vcg = {*
-  Method.no_args (Method.SIMPLE_METHOD' (hoare_tac (K all_tac))) *}
+  Method.ctxt_args (fn ctxt => Method.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 (asm_full_simp_tac (local_simpset_of ctxt)))) *}
+    Method.SIMPLE_METHOD' (hoare_tac ctxt (asm_full_simp_tac (local_simpset_of ctxt)))) *}
   "verification condition generator plus simplification"
 
 end