diff -r 95df71c3df2f -r 3764ed518ee5 Nominal/Nominal2_FSet.thy --- a/Nominal/Nominal2_FSet.thy Thu Apr 08 09:12:13 2010 +0200 +++ b/Nominal/Nominal2_FSet.thy Thu Apr 08 09:13:36 2010 +0200 @@ -24,23 +24,13 @@ is "permute :: perm \ 'a list \ 'a list" -lemma permute_list_zero: "0 \ (x :: 'a list) = x" - by (rule permute_zero) - -lemma permute_fset_zero: "0 \ (x :: 'a fset) = x" - by (lifting permute_list_zero) - -lemma permute_list_plus: "(p + q) \ (x :: 'a list) = p \ q \ x" - by (rule permute_plus) - -lemma permute_fset_plus: "(p + q) \ (x :: 'a fset) = p \ q \ x" - by (lifting permute_list_plus) - -instance - apply default - apply (rule permute_fset_zero) - apply (rule permute_fset_plus) - done +instance proof + fix x :: "'a fset" and p q :: "perm" + show "0 \ x = x" + by (lifting permute_zero [where 'a="'a list"]) + show "(p + q) \ x = p \ q \ x" + by (lifting permute_plus [where 'a="'a list"]) +qed end