src/HOLCF/ex/dagstuhl.thy
author paulson
Wed, 04 Nov 1998 13:00:15 +0100
changeset 5801 d2c97ca3be62
parent 299 febeb36a4ba4
permissions -rw-r--r--
Some streamlining of text. Theory library is now assumed to be LOCAL and not at TUM.

(*
    ID:         $ $
*)

Dagstuhl  =  Stream2 +

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

rules

YS_def    "YS  = fix[LAM x. scons[y][x]]"
YYS_def   "YYS = fix[LAM z. scons[y][scons[y][z]]]"
  
end