src/HOL/Big_Operators.thy
changeset 53374 a14d2a854c02
parent 53174 71a2702da5e0
child 54147 97a8ff4e4ac9
--- a/src/HOL/Big_Operators.thy	Tue Sep 03 00:51:08 2013 +0200
+++ b/src/HOL/Big_Operators.thy	Tue Sep 03 01:12:40 2013 +0200
@@ -46,7 +46,7 @@
 proof -
   from `x \<in> A` obtain B where A: "A = insert x B" and "x \<notin> B"
     by (auto dest: mk_disjoint_insert)
-  moreover from `finite A` this have "finite B" by simp
+  moreover from `finite A` A have "finite B" by simp
   ultimately show ?thesis by simp
 qed