src/HOL/Predicate_Compile_Examples/Examples.thy
changeset 67443 3abf6a722518
parent 66453 cc19f7ca2ed6
child 80914 d97fdabd9e2b
--- a/src/HOL/Predicate_Compile_Examples/Examples.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Predicate_Compile_Examples/Examples.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -235,7 +235,7 @@
 
 type_synonym vname = nat
 type_synonym vvalue = int
-type_synonym var_assign = "vname \<Rightarrow> vvalue"  \<comment>"variable assignment"
+type_synonym var_assign = "vname \<Rightarrow> vvalue"  \<comment> \<open>variable assignment\<close>
 
 datatype ir_expr = 
   IrConst vvalue
@@ -264,7 +264,7 @@
 
 subsection \<open>Another semantics\<close>
 
-type_synonym name = nat \<comment>"For simplicity in examples"
+type_synonym name = nat \<comment> \<open>For simplicity in examples\<close>
 type_synonym state' = "name \<Rightarrow> nat"
 
 datatype aexp = N nat | V name | Plus aexp aexp