src/HOL/HOLCF/IOA/ABP/Env.thy
changeset 62002 f1599e98c4d0
parent 61032 b57df8eecad6
child 62008 cbedaddc9351
--- a/src/HOL/HOLCF/IOA/ABP/Env.thy	Wed Dec 30 21:56:12 2015 +0100
+++ b/src/HOL/HOLCF/IOA/ABP/Env.thy	Wed Dec 30 21:57:52 2015 +0100
@@ -2,14 +2,14 @@
     Author:     Olaf Müller
 *)
 
-section {* The environment *}
+section \<open>The environment\<close>
 
 theory Env
 imports "~~/src/HOL/HOLCF/IOA/meta_theory/IOA" Action
 begin
 
 type_synonym
-  'm env_state = bool   -- {* give next bit to system *}
+  'm env_state = bool   \<comment> \<open>give next bit to system\<close>
 
 definition
   env_asig :: "'m action signature" where