src/HOL/UNITY/Simple/Network.thy
author wenzelm
Wed, 05 Dec 2001 03:19:47 +0100
changeset 12387 fe2353a8d1e8
parent 11195 65ede8dfe304
child 13785 e2fcd88be55d
permissions -rw-r--r--
fixed intro steps;

(*  Title:      HOL/UNITY/Network
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

The Communication Network

From Misra, "A Logic for Concurrent Programming" (1994), section 5.7
*)

Network = UNITY +

(*The state assigns a number to each process variable*)

datatype pvar = Sent | Rcvd | Idle

datatype pname = Aproc | Bproc

types state = "pname * pvar => nat"

end