diff -r b33b42211bbf -r 188826f1ccdb Nominal/Nominal2_Base.thy --- a/Nominal/Nominal2_Base.thy Thu Mar 13 09:30:26 2014 +0000 +++ b/Nominal/Nominal2_Base.thy Mon Mar 24 15:31:17 2014 +0000 @@ -2167,7 +2167,7 @@ proof - have "(\{supp x | x. x \# M}) = (\{supp x | x. x \ set_of M})" by simp also have "... \ (\x \ set_of M. supp x)" by auto - also have "... = supp (set_of M)" by (simp add: subst supp_of_finite_sets) + also have "... = supp (set_of M)" by (simp add: supp_of_finite_sets) also have " ... \ supp M" by (rule supp_set_of) finally show "(\{supp x | x. x \# M}) \ supp M" . qed