src/HOLCF/explicit_domains/Dagstuhl.thy
author paulson
Thu, 18 Jan 1996 10:38:29 +0100
changeset 1444 23ceb1dc9755
parent 1274 ea0668a1c0ba
child 1479 21eb5e156d91
permissions -rw-r--r--
trivial updates

(* $Id$ *)


Dagstuhl  =  Stream2 +

consts
	y  :: "'a"
       YS  :: "'a stream"
       YYS :: "'a stream"

defs

YS_def    "YS  == fix`(LAM x. scons`y`x)"
YYS_def   "YYS == fix`(LAM z. scons`y`(scons`y`z))"
  
end