1
(* Title: HOLCF/IOA/meta_theory/IOA.thy
2
ID: $Id$
3
Author: Olaf Müller
4
*)
5
6
header {* The theory of I/O automata in HOLCF *}
7
8
theory IOA
9
imports SimCorrectness Compositionality Deadlock
10
begin
11
12
end