| 3807 |      1 | (* 
 | 
|  |      2 |     File:        RPCMemoryParams.thy
 | 
|  |      3 |     Author:      Stephan Merz
 | 
|  |      4 |     Copyright:   1997 University of Munich
 | 
|  |      5 | 
 | 
|  |      6 |     Theory Name: RPCMemoryParams
 | 
|  |      7 |     Logic Image: TLA
 | 
|  |      8 | 
 | 
|  |      9 |     Basic declarations for the RPC-memory example.
 | 
|  |     10 | *)
 | 
|  |     11 | 
 | 
| 11703 |     12 | theory RPCMemoryParams = Main:
 | 
| 3807 |     13 | 
 | 
|  |     14 | types
 | 
| 6255 |     15 |   bit = "bool"   (* Signal wires for the procedure interface.
 | 
|  |     16 |                     Defined as bool for simplicity. All I should really need is
 | 
|  |     17 |                     the existence of two distinct values. *)
 | 
| 3807 |     18 | 
 | 
|  |     19 | (* all of these are simple (HOL) types *)
 | 
| 11703 |     20 | typedecl Locs    (* "syntactic" value type *)
 | 
|  |     21 | typedecl Vals    (* "syntactic" value type *)
 | 
|  |     22 | typedecl PrIds   (* process id's *)
 | 
| 3807 |     23 | 
 | 
|  |     24 | end
 |