src/HOLCF/explicit_domains/Dagstuhl.thy
author oheimb
Wed, 18 Dec 1996 15:16:13 +0100
changeset 2445 51993fea433f
parent 1479 21eb5e156d91
permissions -rw-r--r--
removed Holcfb.thy and Holcfb.ML, moving classical3 to HOL.ML as classical2

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