src/HOLCF/explicit_domains/Dagstuhl.thy
author paulson
Mon, 23 Sep 1996 17:42:56 +0200
changeset 2003 b48f066d52dc
parent 1479 21eb5e156d91
permissions -rw-r--r--
Addition of gensym

(* $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