src/HOLCF/FOCUS/FOCUS.thy
changeset 17293 ecf182ccc3ca
parent 14981 e73f8140af78
child 19759 2d0896653e7a
--- a/src/HOLCF/FOCUS/FOCUS.thy	Tue Sep 06 20:53:27 2005 +0200
+++ b/src/HOLCF/FOCUS/FOCUS.thy	Tue Sep 06 21:51:17 2005 +0200
@@ -1,8 +1,12 @@
-(*  Title: 	HOLCF/FOCUS/FOCUS.thy
+(*  Title:      HOLCF/FOCUS/FOCUS.thy
     ID:         $Id$
-    Author: 	David von Oheimb, TU Muenchen
-
-top level of FOCUS
+    Author:     David von Oheimb, TU Muenchen
 *)
 
-FOCUS = Fstream
+header {* Top level of FOCUS *}
+
+theory FOCUS
+imports Fstream
+begin
+
+end