src/HOL/Nominal/Nominal.thy
changeset 41550 efa734d9b221
parent 41413 64cd30d6b0b8
child 41562 90fb3d7474df
--- a/src/HOL/Nominal/Nominal.thy	Fri Jan 14 15:43:04 2011 +0100
+++ b/src/HOL/Nominal/Nominal.thy	Fri Jan 14 15:44:47 2011 +0100
@@ -785,7 +785,7 @@
   hence "((UNIV::'x set) - A) \<noteq> ({}::'x set)" by (force simp only:)
   then obtain c::"'x" where "c\<in>((UNIV::'x set) - A)" by force
   then have "c\<notin>A" by simp
-  then show ?thesis using prems by simp 
+  then show ?thesis ..
 qed
 
 text {* there always exists a fresh name for an object with finite support *}