src/HOL/IMP/Vars.thy
changeset 67406 23307fd33906
parent 58889 5b7a9633cfa8
child 69505 cc2d676d5395
--- a/src/HOL/IMP/Vars.thy	Thu Jan 11 13:48:17 2018 +0100
+++ b/src/HOL/IMP/Vars.thy	Fri Jan 12 14:08:53 2018 +0100
@@ -7,17 +7,17 @@
 
 subsection "The Variables in an Expression"
 
-text{* We need to collect the variables in both arithmetic and boolean
+text\<open>We need to collect the variables in both arithmetic and boolean
 expressions. For a change we do not introduce two functions, e.g.\ @{text
 avars} and @{text bvars}, but we overload the name @{text vars}
-via a \emph{type class}, a device that originated with Haskell: *}
+via a \emph{type class}, a device that originated with Haskell:\<close>
  
 class vars =
 fixes vars :: "'a \<Rightarrow> vname set"
 
-text{* This defines a type class ``vars'' with a single
+text\<open>This defines a type class ``vars'' with a single
 function of (coincidentally) the same name. Then we define two separated
-instances of the class, one for @{typ aexp} and one for @{typ bexp}: *}
+instances of the class, one for @{typ aexp} and one for @{typ bexp}:\<close>
 
 instantiation aexp :: vars
 begin