diff -r dd58f13a8eb4 -r eb85850d3eb7 src/ZF/Constructible/Normal.thy --- a/src/ZF/Constructible/Normal.thy Fri Nov 17 02:19:55 2006 +0100 +++ b/src/ZF/Constructible/Normal.thy Fri Nov 17 02:20:03 2006 +0100 @@ -19,13 +19,15 @@ subsection {*Closed and Unbounded (c.u.) Classes of Ordinals*} definition - Closed :: "(i=>o) => o" + Closed :: "(i=>o) => o" where "Closed(P) == \I. I \ 0 --> (\i\I. Ord(i) \ P(i)) --> P(\(I))" - Unbounded :: "(i=>o) => o" +definition + Unbounded :: "(i=>o) => o" where "Unbounded(P) == \i. Ord(i) --> (\j. i P(j))" - Closed_Unbounded :: "(i=>o) => o" +definition + Closed_Unbounded :: "(i=>o) => o" where "Closed_Unbounded(P) == Closed(P) \ Unbounded(P)" @@ -201,16 +203,19 @@ subsection {*Normal Functions*} definition - mono_le_subset :: "(i=>i) => o" + mono_le_subset :: "(i=>i) => o" where "mono_le_subset(M) == \i j. i\j --> M(i) \ M(j)" - mono_Ord :: "(i=>i) => o" +definition + mono_Ord :: "(i=>i) => o" where "mono_Ord(F) == \i j. i F(i) < F(j)" - cont_Ord :: "(i=>i) => o" +definition + cont_Ord :: "(i=>i) => o" where "cont_Ord(F) == \l. Limit(l) --> F(l) = (\ii) => o" +definition + Normal :: "(i=>i) => o" where "Normal(F) == mono_Ord(F) \ cont_Ord(F)" @@ -373,7 +378,7 @@ normal function, by @{thm [source] Normal_imp_fp_Unbounded}. *} definition - normalize :: "[i=>i, i] => i" + normalize :: "[i=>i, i] => i" where "normalize(F,a) == transrec2(a, F(0), \x r. F(succ(x)) Un succ(r))" @@ -425,7 +430,7 @@ numbers.*} definition - Aleph :: "i => i" + Aleph :: "i => i" where "Aleph(a) == transrec2(a, nat, \x r. csucc(r))" notation (xsymbols)