src/HOLCF/ex/Dnat.thy
changeset 16417 9bc16273c2d4
parent 16322 7cd7d21975ad
child 19550 ae77a20f6995
--- a/src/HOLCF/ex/Dnat.thy	Fri Jun 17 11:35:35 2005 +0200
+++ b/src/HOLCF/ex/Dnat.thy	Fri Jun 17 16:12:49 2005 +0200
@@ -5,7 +5,7 @@
 Theory for the domain of natural numbers  dnat = one ++ dnat
 *)
 
-theory Dnat = HOLCF:
+theory Dnat imports HOLCF begin
 
 domain dnat = dzero | dsucc (dpred :: dnat)