src/HOL/MicroJava/DFA/Kildall.thy
changeset 67443 3abf6a722518
parent 66453 cc19f7ca2ed6
child 67613 ce654b0e6d69
--- a/src/HOL/MicroJava/DFA/Kildall.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/MicroJava/DFA/Kildall.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -348,10 +348,10 @@
  r = "{(ss',ss) . ss <[r] ss'} <*lex*> finite_psubset"
        in while_rule)
 
-\<comment> "Invariant holds initially:"
+\<comment> \<open>Invariant holds initially:\<close>
 apply (simp add:stables_def)
 
-\<comment> "Invariant is preserved:"
+\<comment> \<open>Invariant is preserved:\<close>
 apply(simp add: stables_def split_paired_all)
 apply(rename_tac ss w)
 apply(subgoal_tac "(SOME p. p \<in> w) \<in> w")
@@ -393,16 +393,16 @@
 apply (blast dest!: boundedD)
 
 
-\<comment> "Postcondition holds upon termination:"
+\<comment> \<open>Postcondition holds upon termination:\<close>
 apply(clarsimp simp add: stables_def split_paired_all)
 
-\<comment> "Well-foundedness of the termination relation:"
+\<comment> \<open>Well-foundedness of the termination relation:\<close>
 apply (rule wf_lex_prod)
  apply (insert orderI [THEN acc_le_listI])
  apply (simp add: acc_def lesssub_def wfP_wf_eq [symmetric])
 apply (rule wf_finite_psubset) 
 
-\<comment> "Loop decreases along termination relation:"
+\<comment> \<open>Loop decreases along termination relation:\<close>
 apply(simp add: stables_def split_paired_all)
 apply(rename_tac ss w)
 apply(subgoal_tac "(SOME p. p \<in> w) \<in> w")