src/ZF/UNITY/Distributor.thy
changeset 60770 240563fbf41d
parent 59788 6f7b6adac439
child 61798 27f3c10b0b50
--- a/src/ZF/UNITY/Distributor.thy	Thu Jul 23 14:20:51 2015 +0200
+++ b/src/ZF/UNITY/Distributor.thy	Thu Jul 23 14:25:05 2015 +0200
@@ -8,9 +8,9 @@
 
 theory Distributor imports AllocBase Follows  Guar GenPrefix begin
 
-text{*Distributor specification (the number of outputs is Nclients)*}
+text\<open>Distributor specification (the number of outputs is Nclients)\<close>
 
-text{*spec (14)*}
+text\<open>spec (14)\<close>
 
 definition
   distr_follows :: "[i, i, i, i =>i] =>i"  where
@@ -37,10 +37,10 @@
      distr_follows(A, In, iIn, Out) \<inter> distr_allowed_acts(Out)"
 
 locale distr =
-  fixes In  --{*items to distribute*}
-    and iIn --{*destinations of items to distribute*}
-    and Out --{*distributed items*}
-    and A   --{*the type of items being distributed *}
+  fixes In  --\<open>items to distribute\<close>
+    and iIn --\<open>destinations of items to distribute\<close>
+    and Out --\<open>distributed items\<close>
+    and A   --\<open>the type of items being distributed\<close>
     and D
  assumes
      var_assumes [simp]:  "In \<in> var & iIn \<in> var & (\<forall>n. Out(n):var)"