diff -r 266abc3ee228 -r 99367d481f78 Nominal/FSet.thy --- a/Nominal/FSet.thy Thu Apr 22 12:33:51 2010 +0200 +++ b/Nominal/FSet.thy Thu Apr 22 12:42:15 2010 +0200 @@ -1070,7 +1070,8 @@ "(finsert x xs |\| ys) = (x |\| ys \ xs |\| ys)" by (lifting sub_list_cons) -thm sub_list_def[simplified memb_def[symmetric], quot_lifted, no_vars] +lemma "xs |\| ys \ \x. x |\| xs \ x |\| ys" + by (lifting sub_list_def[simplified memb_def[symmetric]]) lemma fsubset_fin: "xs |\| ys = (\x. x |\| xs \ x |\| ys)" by (rule meta_eq_to_obj_eq)