src/HOL/MicroJava/BV/BVSpecTypeSafe.thy
changeset 13672 b95d12325b51
parent 13524 604d0f3622d6
child 13678 c748d11547d8
equal deleted inserted replaced
13671:eec2582923f6 13672:b95d12325b51
   240     with cr' match phi' meth  
   240     with cr' match phi' meth  
   241     show ?thesis by (unfold correct_state_def) auto
   241     show ?thesis by (unfold correct_state_def) auto
   242   qed
   242   qed
   243 qed
   243 qed
   244 
   244 
   245 
   245 declare raise_if_def [simp]
   246 text {*
   246 text {*
   247   The requirement of lemma @{text uncaught_xcpt_correct} (that
   247   The requirement of lemma @{text uncaught_xcpt_correct} (that
   248   the exception is a valid reference on the heap) is always met
   248   the exception is a valid reference on the heap) is always met
   249   for welltyped instructions and conformant states:
   249   for welltyped instructions and conformant states:
   250 *}
   250 *}