src/HOLCF/ex/Stream.thy
author wenzelm
Sun, 25 Oct 1998 12:33:27 +0100
changeset 5769 6a422b22ba02
parent 4122 f63c283cefaf
child 9169 85a47aa21f74
permissions -rw-r--r--
tuned checklist;

(*  Title: 	FOCUS/Stream.thy
    ID:         $ $
    Author: 	Franz Regensburger, David von Oheimb
    Copyright   1993, 1995 Technische Universitaet Muenchen

general Stream domain
*)

Stream = HOLCF + 

domain 'a stream = "&&" (ft::'a) (lazy rt::'a stream) (infixr 65)

end