src/HOL/Metis_Examples/Big_O.thy
changeset 63918 6bf55e6e0b75
parent 63167 0909deb8059b
child 64267 b9a1486e79be
--- a/src/HOL/Metis_Examples/Big_O.thy	Mon Sep 19 12:53:30 2016 +0200
+++ b/src/HOL/Metis_Examples/Big_O.thy	Mon Sep 19 20:06:21 2016 +0200
@@ -499,7 +499,7 @@
 apply (subst abs_of_nonneg) back back
  apply (rule setsum_nonneg)
  apply force
-apply (subst setsum_right_distrib)
+apply (subst setsum_distrib_left)
 apply (rule allI)
 apply (rule order_trans)
  apply (rule setsum_abs)