src/HOL/TLA/Memory/MemoryImplementation.thy
changeset 9517 f58863b1406a
parent 6255 db63752140c7
child 11703 6e5de8d4290a
--- a/src/HOL/TLA/Memory/MemoryImplementation.thy	Thu Aug 03 19:28:37 2000 +0200
+++ b/src/HOL/TLA/Memory/MemoryImplementation.thy	Thu Aug 03 19:29:03 2000 +0200
@@ -33,9 +33,6 @@
   rst           :: "rpcStType"
   cst           :: "mClkStType"
   ires          :: "resType"
-(* the history variable : not defined as a constant
-  rmhist        :: "histType"
-*)
 
 constdefs
   (* auxiliary predicates *)
@@ -78,7 +75,7 @@
                            & [][HNext rmhist p]_(c p,r p,m p, rmhist!p)"
 
   Hist          :: "histType => temporal"
-      "Hist rmhist == TEMP (!p. HistP rmhist p)"
+      "Hist rmhist == TEMP (ALL p. HistP rmhist p)"
 
   (* the implementation *)
   IPImp          :: "PrIds => temporal"
@@ -86,7 +83,7 @@
 	               & MClkIPSpec memCh crCh cst p
   	               & RPCIPSpec crCh rmCh rst p
 	               & RPSpec rmCh mm ires p
-		       & (! l. #l : #MemLoc --> MSpec rmCh mm ires l))"
+		       & (ALL l. #l : #MemLoc --> MSpec rmCh mm ires l))"
 
   ImpInit        :: "PrIds => stpred"
       "ImpInit p == PRED (  ~Calling memCh p
@@ -108,7 +105,7 @@
 			& WF(MemReturn rmCh ires p)_(m p)"
 
   Implementation :: "temporal"
-      "Implementation == TEMP ( (!p. Init (~Calling memCh p) & [][ENext p]_(e p))
+      "Implementation == TEMP ( (ALL p. Init (~Calling memCh p) & [][ENext p]_(e p))
                                & MClkISpec memCh crCh cst
                                & RPCISpec crCh rmCh rst
                                & IRSpec rmCh mm ires)"