src/HOL/Library/Binomial.thy
changeset 55158 39bcdf19dd14
parent 55143 04448228381d
--- a/src/HOL/Library/Binomial.thy	Mon Jan 27 16:38:52 2014 +0000
+++ b/src/HOL/Library/Binomial.thy	Mon Jan 27 17:13:33 2014 +0000
@@ -131,7 +131,7 @@
          prefer 4 apply (force simp add: constr_bij)
         prefer 3 apply force
        prefer 2 apply (blast intro: finite_Pow_iff [THEN iffD2]
-         finite_subset [of _ "Pow (insert x F)", standard])
+         finite_subset [of _ "Pow (insert x F)" for F])
       apply (blast intro: finite_Pow_iff [THEN iffD2, THEN [2] finite_subset])
       done
   qed