diff -r 4135198bbb8a -r 56cebe7f8e24 Nominal/FSet.thy --- a/Nominal/FSet.thy Tue Apr 13 00:47:57 2010 +0200 +++ b/Nominal/FSet.thy Tue Apr 13 00:53:32 2010 +0200 @@ -43,8 +43,7 @@ quotient_definition fin ("_ |\| _" [50, 51] 50) where - "fin :: 'a \ 'a fset \ bool" -is "memb" + "fin :: 'a \ 'a fset \ bool" is "memb" abbreviation fnotin :: "'a \ 'a fset \ bool" ("_ |\| _" [50, 51] 50) @@ -63,7 +62,7 @@ shows "(op = ===> op \ ===> op \) op # op #" by simp -section {* Augmenting a set -- @{const finsert} *} +section {* Augmenting an fset -- @{const finsert} *} lemma nil_not_cons: shows