diff -r 7085ab735de7 -r 56b8d977d1c0 Nominal/Atoms.thy --- a/Nominal/Atoms.thy Mon Mar 14 16:35:59 2011 +0100 +++ b/Nominal/Atoms.thy Tue Mar 15 00:40:39 2011 +0100 @@ -80,6 +80,25 @@ This does not work for multi-sorted atoms. *} +(* fixme +lemma supp_of_finite_name_set: + fixes S::"name set" + assumes "infinte S" "infinite (UNIV - S)" + shows "supp S = UNIV" +proof - + { fix a + have "a \ supp S" + proof (cases "a \ atom ` S") + assume "a \ atom ` S" + then have "\b \ UNIV - S. (a \ atom b) \ S \ S" + apply(clarify) + + show "a \ supp S" + } + then show "supp S = UNIV" by auto +qed +*) + section {* Automatic instantiation of class @{text at}. *}