src/HOLCF/HOLCF.thy
changeset 15650 b37dc98fbbc5
parent 15576 efb95d0d01f7
child 15651 4b393520846e
--- a/src/HOLCF/HOLCF.thy	Fri Apr 01 23:44:41 2005 +0200
+++ b/src/HOLCF/HOLCF.thy	Sat Apr 02 00:12:38 2005 +0200
@@ -5,4 +5,8 @@
 Top theory for HOLCF system.
 *)
 
-HOLCF = Sprod + Ssum + Up + Lift + Discrete + One + Tr
+theory HOLCF
+imports Sprod Ssum Up Lift Discrete One Tr
+begin
+
+end