src/HOL/UNITY/Comp/Alloc.thy
changeset 15074 277b3a4da341
parent 11786 51ce34ef5113
child 17310 1322ed8e0ee4
--- a/src/HOL/UNITY/Comp/Alloc.thy	Thu Jul 22 12:55:36 2004 +0200
+++ b/src/HOL/UNITY/Comp/Alloc.thy	Thu Jul 22 17:37:31 2004 +0200
@@ -52,8 +52,8 @@
   (*spec (1)*)
   system_safety :: 'a systemState program set
     "system_safety ==
-     Always {s. (\\<Sum>i: lessThan Nclients. (tokens o giv o sub i o client)s)
-     <= NbT + (\\<Sum>i: lessThan Nclients. (tokens o rel o sub i o client)s)}"
+     Always {s. (SUM i: lessThan Nclients. (tokens o giv o sub i o client)s)
+     <= NbT + (SUM i: lessThan Nclients. (tokens o rel o sub i o client)s)}"
 
   (*spec (2)*)
   system_progress :: 'a systemState program set
@@ -111,8 +111,8 @@
     "alloc_safety ==
 	 (INT i : lessThan Nclients. Increasing (sub i o allocRel))
          guarantees
-	 Always {s. (\\<Sum>i: lessThan Nclients. (tokens o sub i o allocGiv)s)
-         <= NbT + (\\<Sum>i: lessThan Nclients. (tokens o sub i o allocRel)s)}"
+	 Always {s. (SUM i: lessThan Nclients. (tokens o sub i o allocGiv)s)
+         <= NbT + (SUM i: lessThan Nclients. (tokens o sub i o allocRel)s)}"
 
   (*spec (8)*)
   alloc_progress :: 'a allocState_d program set