src/HOL/Unix/Unix.thy
changeset 67443 3abf6a722518
parent 66453 cc19f7ca2ed6
child 68451 c34aa23a1fb6
--- a/src/HOL/Unix/Unix.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/Unix/Unix.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -73,7 +73,7 @@
 datatype perm =
     Readable
   | Writable
-  | Executable    \<comment> "(ignored)"
+  | Executable    \<comment> \<open>(ignored)\<close>
 
 type_synonym perms = "perm set"
 
@@ -875,11 +875,11 @@
   apply (unfold bogus_def bogus_path_def)
   apply (drule transitions_consD, rule transition.intros,
       (force simp add: eval)+, (simp add: eval)?)+
-    \<comment> "evaluate all operations"
+    \<comment> \<open>evaluate all operations\<close>
   apply (drule transitions_nilD)
-    \<comment> "reach final result"
+    \<comment> \<open>reach final result\<close>
   apply (simp add: invariant_def eval)
-    \<comment> "check the invariant"
+    \<comment> \<open>check the invariant\<close>
   done
 
 text \<open>