src/HOL/MicroJava/DFA/Typing_Framework_err.thy
changeset 69597 ff784d5a5bfb
parent 63170 eae6549dbea2
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   159 
   159 
   160 
   160 
   161 text \<open>
   161 text \<open>
   162   There used to be a condition here that each instruction must have a
   162   There used to be a condition here that each instruction must have a
   163   successor. This is not needed any more, because the definition of
   163   successor. This is not needed any more, because the definition of
   164   @{term error} trivially ensures that there is a successor for
   164   \<^term>\<open>error\<close> trivially ensures that there is a successor for
   165   the critical case where @{term app} does not hold. 
   165   the critical case where \<^term>\<open>app\<close> does not hold. 
   166 \<close>
   166 \<close>
   167 lemma wt_err_imp_wt_app_eff:
   167 lemma wt_err_imp_wt_app_eff:
   168   assumes wt: "wt_err_step r (err_step (size ts) app step) ts"
   168   assumes wt: "wt_err_step r (err_step (size ts) app step) ts"
   169   assumes b:  "bounded (err_step (size ts) app step) (size ts)"
   169   assumes b:  "bounded (err_step (size ts) app step) (size ts)"
   170   shows "wt_app_eff r app step (map ok_val ts)"
   170   shows "wt_app_eff r app step (map ok_val ts)"