src/HOL/Analysis/Homeomorphism.thy
changeset 63918 6bf55e6e0b75
parent 63627 6ddb43c6b711
child 63945 444eafb6e864
--- a/src/HOL/Analysis/Homeomorphism.thy	Mon Sep 19 12:53:30 2016 +0200
+++ b/src/HOL/Analysis/Homeomorphism.thy	Mon Sep 19 20:06:21 2016 +0200
@@ -1007,7 +1007,7 @@
   have gf[simp]: "g (f x) = x" for x
     apply (rule euclidean_eqI)
     apply (simp add: f_def g_def inner_setsum_left scaleR_setsum_left algebra_simps)
-    apply (simp add: Groups_Big.setsum_right_distrib [symmetric] *)
+    apply (simp add: Groups_Big.setsum_distrib_left [symmetric] *)
     done
   then have "inj f" by (metis injI)
   have gfU: "g ` f ` U = U"