src/HOL/IMP/Def_Init_Big.thy
changeset 67406 23307fd33906
parent 53015 a1119cf551e8
child 69597 ff784d5a5bfb
--- a/src/HOL/IMP/Def_Init_Big.thy	Thu Jan 11 13:48:17 2018 +0100
+++ b/src/HOL/IMP/Def_Init_Big.thy	Fri Jan 12 14:08:53 2018 +0100
@@ -32,8 +32,8 @@
 
 subsection "Soundness wrt Big Steps"
 
-text{* Note the special form of the induction because one of the arguments
-of the inductive predicate is not a variable but the term @{term"Some s"}: *}
+text\<open>Note the special form of the induction because one of the arguments
+of the inductive predicate is not a variable but the term @{term"Some s"}:\<close>
 
 theorem Sound:
   "\<lbrakk> (c,Some s) \<Rightarrow> s';  D A c A';  A \<subseteq> dom s \<rbrakk>
@@ -55,7 +55,7 @@
     by auto (metis bval_Some option.simps(3) order_trans)
 next
   case (WhileTrue b s c s' s'')
-  from `D A (WHILE b DO c) A'` obtain A' where "D A c A'" by blast
+  from \<open>D A (WHILE b DO c) A'\<close> obtain A' where "D A c A'" by blast
   then obtain t' where "s' = Some t'" "A \<subseteq> dom t'"
     by (metis D_incr WhileTrue(3,7) subset_trans)
   from WhileTrue(5)[OF this(1) WhileTrue(6) this(2)] show ?case .