src/HOL/Finite_Set.thy
changeset 27611 2c01c0bdb385
parent 27430 1e25ac05cd87
child 27981 feb0c01cf0fb
--- a/src/HOL/Finite_Set.thy	Tue Jul 15 16:02:10 2008 +0200
+++ b/src/HOL/Finite_Set.thy	Tue Jul 15 16:50:09 2008 +0200
@@ -753,11 +753,14 @@
 *}
 
 lemma fold_fusion:
-  includes ab_semigroup_mult g
+  assumes "ab_semigroup_mult g"
   assumes fin: "finite A"
     and hyp: "\<And>x y. h (g x y) = times x (h y)"
   shows "h (fold g j w A) = fold times j (h w) A"
-  using fin hyp by (induct set: finite) simp_all
+proof -
+  interpret ab_semigroup_mult [g] by fact
+  show ?thesis using fin hyp by (induct set: finite) simp_all
+qed
 
 lemma fold_cong:
   "finite A \<Longrightarrow> (!!x. x:A ==> g x = h x) ==> fold times g z A = fold times h z A"