src/HOL/Integration.thy
changeset 33640 0d82107dc07a
parent 32960 69916a850301
--- a/src/HOL/Integration.thy	Thu Nov 12 17:21:48 2009 +0100
+++ b/src/HOL/Integration.thy	Thu Nov 12 17:21:51 2009 +0100
@@ -542,7 +542,7 @@
  apply (erule subst)
  apply (subst listsum_subtractf [symmetric])
  apply (rule listsum_abs [THEN order_trans])
- apply (subst map_compose [symmetric, unfolded o_def])
+ apply (subst map_map [unfolded o_def])
  apply (subgoal_tac "e = (\<Sum>(u, x, v)\<leftarrow>D. (e / (b - a)) * (v - u))")
   apply (erule ssubst)
   apply (simp add: abs_minus_commute)