src/HOL/TLA/Memory/MemoryParameters.thy
changeset 9517 f58863b1406a
parent 6255 db63752140c7
child 17309 c43ed29bd197
--- a/src/HOL/TLA/Memory/MemoryParameters.thy	Thu Aug 03 19:28:37 2000 +0200
+++ b/src/HOL/TLA/Memory/MemoryParameters.thy	Thu Aug 03 19:29:03 2000 +0200
@@ -12,19 +12,8 @@
 MemoryParameters = Datatype + RPCMemoryParams +
 
 (* the memory operations *)
-(***
-datatype  Rd = read
-datatype  Wr = write
-***)
-
 datatype memOp = read Locs | write Locs Vals
 
-(***
-types
-  (* legal arguments for the memory *)
-  memArgType = "(Rd * Locs) + (Wr * Locs * Vals)"
-***)
-
 consts
   (* memory locations and contents *)
   MemLoc         :: Locs set