src/HOLCF/ex/Stream.thy
author paulson
Fri, 25 Aug 2000 12:15:35 +0200
changeset 9687 772ac061bd76
parent 9169 85a47aa21f74
child 11348 e08a0855af67
permissions -rw-r--r--
moved congruence rules UN_cong, INT_cong from UNTIY/Union to Set.ML

(*  Title: 	HOLCF/ex//Stream.thy
    ID:         $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