src/HOLCF/ex/Dagstuhl.thy
changeset 17291 94f6113fe9ed
parent 10835 f4745d77e620
child 19742 86f21beabafc
--- a/src/HOLCF/ex/Dagstuhl.thy	Tue Sep 06 19:22:31 2005 +0200
+++ b/src/HOLCF/ex/Dagstuhl.thy	Tue Sep 06 19:28:58 2005 +0200
@@ -1,17 +1,19 @@
 (* $Id$ *)
 
-
-Dagstuhl  =  Stream +
+theory Dagstuhl
+imports Stream
+begin
 
 consts
-        y  :: "'a"
-       YS  :: "'a stream"
-       YYS :: "'a stream"
+  y  :: "'a"
 
-defs
+constdefs
+  YS :: "'a stream"
+  "YS == fix$(LAM x. y && x)"
+  YYS :: "'a stream"
+  "YYS == fix$(LAM z. y && y && z)"
 
-YS_def    "YS  == fix$(LAM x. y && x)"
-YYS_def   "YYS == fix$(LAM z. y && y && z)"
-  
+ML {* use_legacy_bindings (the_context ()) *}
+
 end