author | paulson |
Wed, 05 Aug 1998 10:57:25 +0200 | |
changeset 5253 | 82a5ca6290aa |
parent 5252 | 1b0f14d11142 |
child 5259 | 86d80749453f |
permissions | -rw-r--r-- |
5252 | 1 |
(* Title: HOL/UNITY/Union.thy |
2 |
ID: $Id$ |
|
3 |
Author: Lawrence C Paulson, Cambridge University Computer Laboratory |
|
4 |
Copyright 1998 University of Cambridge |
|
5 |
||
6 |
Unions of programs |
|
7 |
||
8 |
From Misra's Chapter 5: Asynchronous Compositions of Programs |
|
9 |
*) |
|
10 |
||
11 |
Union = SubstAx + FP + |
|
12 |
||
13 |
constdefs |
|
14 |
||
15 |
Join :: "['a program, 'a program] => 'a program" |
|
16 |
"Join prgF prgG == (|Init = Init prgF Int Init prgG, |
|
17 |
Acts = Acts prgF Un Acts prgG|)" |
|
18 |
||
19 |
end |