equal
deleted
inserted
replaced
31 succ :: "['a set set,'a set set] => 'a set set" where |
31 succ :: "['a set set,'a set set] => 'a set set" where |
32 "succ S c = |
32 "succ S c = |
33 (if c \<notin> chain S | c \<in> maxchain S |
33 (if c \<notin> chain S | c \<in> maxchain S |
34 then c else SOME c'. c' \<in> super S c)" |
34 then c else SOME c'. c' \<in> super S c)" |
35 |
35 |
36 consts |
36 inductive_set |
37 TFin :: "'a set set => 'a set set set" |
37 TFin :: "'a set set => 'a set set set" |
38 inductive "TFin S" |
38 for S :: "'a set set" |
39 intros |
39 where |
40 succI: "x \<in> TFin S ==> succ S x \<in> TFin S" |
40 succI: "x \<in> TFin S ==> succ S x \<in> TFin S" |
41 Pow_UnionI: "Y \<in> Pow(TFin S) ==> Union(Y) \<in> TFin S" |
41 | Pow_UnionI: "Y \<in> Pow(TFin S) ==> Union(Y) \<in> TFin S" |
42 monos Pow_mono |
42 monos Pow_mono |
43 |
43 |
44 |
44 |
45 subsection{*Mathematical Preamble*} |
45 subsection{*Mathematical Preamble*} |
46 |
46 |