src/HOL/MicroJava/DFA/Typing_Framework_err.thy
changeset 61361 8b5f00202e1a
parent 58886 8a6cac7c7247
child 61994 133a8a888ae8
--- a/src/HOL/MicroJava/DFA/Typing_Framework_err.thy	Wed Oct 07 19:45:00 2015 +0200
+++ b/src/HOL/MicroJava/DFA/Typing_Framework_err.thy	Wed Oct 07 23:28:49 2015 +0200
@@ -3,7 +3,7 @@
     Copyright   2000 TUM
 *)
 
-section {* Lifting the Typing Framework to err, app, and eff *}
+section \<open>Lifting the Typing Framework to err, app, and eff\<close>
 
 theory Typing_Framework_err
 imports Typing_Framework SemilatAlg
@@ -158,12 +158,12 @@
 
 
 
-text {*
+text \<open>
   There used to be a condition here that each instruction must have a
   successor. This is not needed any more, because the definition of
   @{term error} trivially ensures that there is a successor for
   the critical case where @{term app} does not hold. 
-*}
+\<close>
 lemma wt_err_imp_wt_app_eff:
   assumes wt: "wt_err_step r (err_step (size ts) app step) ts"
   assumes b:  "bounded (err_step (size ts) app step) (size ts)"