src/HOL/Hoare/HoareAbort.thy
changeset 15032 02aed07e01bf
parent 13875 12997e3ddd8d
child 16417 9bc16273c2d4
equal deleted inserted replaced
15031:726dc9146bb1 15032:02aed07e01bf
   243   "verification condition generator"
   243   "verification condition generator"
   244 
   244 
   245 method_setup vcg_simp = {*
   245 method_setup vcg_simp = {*
   246   Method.ctxt_args (fn ctxt =>
   246   Method.ctxt_args (fn ctxt =>
   247     Method.METHOD (fn facts => 
   247     Method.METHOD (fn facts => 
   248       hoare_tac (asm_full_simp_tac (Simplifier.get_local_simpset ctxt))1)) *}
   248       hoare_tac (asm_full_simp_tac (local_simpset_of ctxt))1)) *}
   249   "verification condition generator plus simplification"
   249   "verification condition generator plus simplification"
   250 
   250 
   251 (* Special syntax for guarded statements and guarded array updates: *)
   251 (* Special syntax for guarded statements and guarded array updates: *)
   252 
   252 
   253 syntax
   253 syntax