src/HOL/TLA/Memory/MemoryParameters.thy
changeset 3807 82a99b090d9d
child 5184 9b8547a9496a
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/HOL/TLA/Memory/MemoryParameters.thy	Wed Oct 08 11:50:33 1997 +0200
@@ -0,0 +1,50 @@
+(*
+    File:        MemoryParameters.thy
+    Author:      Stephan Merz
+    Copyright:   1997 University of Munich
+
+    Theory Name: MemoryParameters
+    Logic Image: TLA
+
+    RPC-Memory example: Memory parameters
+*)
+
+MemoryParameters = Prod + Sum + Arith + RPCMemoryParams +
+
+(* the memory operations. nb: data types must be defined in theories
+   that do not include Intensional -- otherwise the induction rule
+   can't be type-checked unambiguously.
+*)
+datatype  Rd = read
+datatype  Wr = write
+
+types
+  (* legal arguments for the memory *)
+  memArgType = "(Rd * Locs) + (Wr * Locs * Vals)"
+
+consts
+  (* memory locations and contents *)
+  MemLoc         :: "Locs => bool"
+  MemVal         :: "Vals => bool"
+
+  (* some particular values *)
+  OK             :: "Vals"
+  BadArg         :: "Vals"
+  MemFailure     :: "Vals"
+  NotAResult     :: "Vals"  (* defined here for simplicity *)
+  
+  (* the initial value stored in each memory cell *)
+  InitVal        :: "Vals"
+
+rules
+  (* basic assumptions about the above constants and predicates *)
+  BadArgNoMemVal    "~MemVal(BadArg)"
+  MemFailNoMemVal   "~MemVal(MemFailure)"
+  InitValMemVal     "MemVal(InitVal)"
+  NotAResultNotVal  "~MemVal(NotAResult)"
+  NotAResultNotOK   "NotAResult ~= OK"
+  NotAResultNotBA   "NotAResult ~= BadArg"
+  NotAResultNotMF   "NotAResult ~= MemFailure"
+end
+
+