diff -r e453c480d599 -r ffc5054a7274 src/HOL/Nominal/Examples/Support.thy --- a/src/HOL/Nominal/Examples/Support.thy Sun Oct 21 19:12:05 2007 +0200 +++ b/src/HOL/Nominal/Examples/Support.thy Sun Oct 21 19:32:19 2007 +0200 @@ -5,17 +5,15 @@ begin text {* - An example showing that in general x\(A \ B) does not imply x\A and x\B - The example shows that with A set to the set of - even atoms and B to the set of odd even atoms. - Then A \ B, that is the set of all atoms, has - empty support. The sets A, respectively B, have - the set of all atoms as support. - + For this we set A to the set of even atoms + and B to the set of odd even atoms. Then A \ B, + that is the set of all atoms, has empty support. + The sets A, respectively B, have the set of all atoms + as support. *} atom_decl atom @@ -37,6 +35,7 @@ lemma EVEN_union_ODD: shows "EVEN \ ODD = UNIV" + using even_or_odd proof - have "EVEN \ ODD = (\n. atom n) ` {n. \i. n = 2*i} \ (\n. atom n) ` {n. \i. n = 2*i+1}" by auto also have "\ = (\n. atom n) ` ({n. \i. n = 2*i} \ {n. \i. n = 2*i+1})" by auto @@ -69,7 +68,9 @@ apply(auto simp add: inj_on_def) done -(* A set S that is infinite and coinfinite has all atoms as its support *) +text {* + A set S that is infinite and coinfinite + has all atoms as its support. *} lemma supp_infinite_coinfinite: fixes S::"atom set" assumes a: "infinite S"