src/HOLCF/IOA/meta_theory/IOA.thy
changeset 17233 41eee2e7b465
parent 14981 e73f8140af78
child 35174 e15040ae75d7
--- a/src/HOLCF/IOA/meta_theory/IOA.thy	Fri Sep 02 15:54:47 2005 +0200
+++ b/src/HOLCF/IOA/meta_theory/IOA.thy	Fri Sep 02 17:23:59 2005 +0200
@@ -1,8 +1,12 @@
 (*  Title:      HOLCF/IOA/meta_theory/IOA.thy
     ID:         $Id$
     Author:     Olaf Müller
+*)
 
-The theory of I/O automata in HOLCF.
-*)   
-	       
-IOA = SimCorrectness + Compositionality + Deadlock
+header {* The theory of I/O automata in HOLCF *}
+
+theory IOA
+imports SimCorrectness Compositionality Deadlock
+begin
+
+end