changeset 0 | 7949f97df77a |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/ex/Rec.thy Thu Sep 16 12:21:07 1993 +0200 @@ -0,0 +1,9 @@ +Rec = Fixedpt + +consts +fix :: "('a=>'a) => 'a" +Dom :: "(('a=>'b) => ('a=>'b)) => 'a set" +Domf :: "(('a=>'b) => ('a=>'b)) => 'a set => 'a set" +rules +Domf_def "Domf(F,D) == {y . !f g. (!x:D. f(x)=g(x)) --> F(f,y)=F(g,y)}" +Dom_def "Dom(F) == lfp(Domf(F))" +end