src/HOLCF/ex/Coind.thy
changeset 1274 ea0668a1c0ba
parent 1273 6960ec882bca
child 1275 5d68da443a9f
--- a/src/HOLCF/ex/Coind.thy	Fri Oct 06 16:17:08 1995 +0100
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,33 +0,0 @@
-(*  Title: 	HOLCF/coind.thy
-    ID:         $Id$
-    Author: 	Franz Regensburger
-    Copyright   1993 Technische Universitaet Muenchen
-
-Example for co-induction on streams
-*)
-
-Coind = Stream2 +
-
-
-consts
-
-	nats		:: "dnat stream"
-	from		:: "dnat -> dnat stream"
-
-defs
-	nats_def	"nats == fix`(LAM h.scons`dzero`(smap`dsucc`h))"
-
-	from_def	"from == fix`(LAM h n.scons`n`(h`(dsucc`n)))"
-
-end
-
-(*
-		smap`f`UU = UU
-      x~=UU --> smap`f`(scons`x`xs) = scons`(f`x)`(smap`f`xs)
-
-		nats = scons`dzero`(smap`dsucc`nats)
-
-		from`n = scons`n`(from`(dsucc`n))
-*)
-
-