1
(* $Id$ *)
2
3
4
Dagstuhl = Stream +
5
6
consts
7
y :: "'a"
8
YS :: "'a stream"
9
YYS :: "'a stream"
10
11
defs
12
13
YS_def "YS == fix$(LAM x. y && x)"
14
YYS_def "YYS == fix$(LAM z. y && y && z)"
15
16
end
17