diff -r 3ca49a4bcc9f -r 38a46e029784 src/HOL/Multivariate_Analysis/Integration.thy --- a/src/HOL/Multivariate_Analysis/Integration.thy Tue Dec 27 09:15:26 2011 +0100 +++ b/src/HOL/Multivariate_Analysis/Integration.thy Tue Dec 27 09:45:10 2011 +0100 @@ -1814,7 +1814,7 @@ unfolding monoidal_def forall_option neutral_lifted[OF assms] using monoidal_ac[OF assms] by auto definition "support opp f s = {x. x\s \ f x \ neutral opp}" -definition "fold' opp e s \ (if finite s then fold opp e s else e)" +definition "fold' opp e s \ (if finite s then Finite_Set.fold opp e s else e)" definition "iterate opp s f \ fold' (\x a. opp (f x) a) (neutral opp) (support opp f s)" lemma support_subset[intro]:"support opp f s \ s" unfolding support_def by auto