src/HOL/Hoare/Hoare.thy
changeset 30549 d2d7874648bd
parent 30510 4120fc59dd85
child 32134 ee143615019c
equal deleted inserted replaced
30548:2eef5e71edd6 30549:d2d7874648bd
   232 
   232 
   233 lemmas AbortRule = SkipRule  -- "dummy version"
   233 lemmas AbortRule = SkipRule  -- "dummy version"
   234 use "hoare_tac.ML"
   234 use "hoare_tac.ML"
   235 
   235 
   236 method_setup vcg = {*
   236 method_setup vcg = {*
   237   Method.ctxt_args (fn ctxt => SIMPLE_METHOD' (hoare_tac ctxt (K all_tac))) *}
   237   Scan.succeed (fn ctxt => SIMPLE_METHOD' (hoare_tac ctxt (K all_tac))) *}
   238   "verification condition generator"
   238   "verification condition generator"
   239 
   239 
   240 method_setup vcg_simp = {*
   240 method_setup vcg_simp = {*
   241   Method.ctxt_args (fn ctxt =>
   241   Scan.succeed (fn ctxt =>
   242     SIMPLE_METHOD' (hoare_tac ctxt (asm_full_simp_tac (local_simpset_of ctxt)))) *}
   242     SIMPLE_METHOD' (hoare_tac ctxt (asm_full_simp_tac (local_simpset_of ctxt)))) *}
   243   "verification condition generator plus simplification"
   243   "verification condition generator plus simplification"
   244 
   244 
   245 end
   245 end