src/HOL/Set.thy
changeset 55143 04448228381d
parent 54998 8601434fa334
child 55775 1557a391a858
--- a/src/HOL/Set.thy	Sat Jan 25 21:52:04 2014 +0100
+++ b/src/HOL/Set.thy	Sat Jan 25 22:06:07 2014 +0100
@@ -1577,10 +1577,10 @@
   by (auto simp add: Pow_def)
 
 lemma Pow_insert: "Pow (insert a A) = Pow A \<union> (insert a ` Pow A)"
-  by (blast intro: image_eqI [where ?x = "u - {a}", standard])
+  by (blast intro: image_eqI [where ?x = "u - {a}" for u])
 
 lemma Pow_Compl: "Pow (- A) = {-B | B. A \<in> Pow B}"
-  by (blast intro: exI [where ?x = "- u", standard])
+  by (blast intro: exI [where ?x = "- u" for u])
 
 lemma Pow_UNIV [simp]: "Pow UNIV = UNIV"
   by blast