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