Instantiated subst rule to avoid problems with HO unification.
authorberghofe
Wed, 07 May 2008 10:56:33 +0200
changeset 26791 3581a9c71909
parent 26790 e8cc166ba123
child 26792 f2d75fd23124
Instantiated subst rule to avoid problems with HO unification.
src/HOL/Equiv_Relations.thy
--- a/src/HOL/Equiv_Relations.thy	Tue May 06 23:33:05 2008 +0200
+++ b/src/HOL/Equiv_Relations.thy	Wed May 07 10:56:33 2008 +0200
@@ -316,7 +316,7 @@
 lemma equiv_imp_dvd_card:
   "finite A ==> equiv A r ==> \<forall>X \<in> A//r. k dvd card X
     ==> k dvd card A"
-  apply (rule Union_quotient [THEN subst])
+  apply (rule Union_quotient [THEN subst [where P="\<lambda>A. k dvd card A"]])
    apply assumption
   apply (rule dvd_partition)
      prefer 3 apply (blast dest: quotient_disj)