diff -r c09598a97436 -r d8d85a8172b5 src/HOL/Inequalities.thy --- a/src/HOL/Inequalities.thy Sat Jul 18 21:44:18 2015 +0200 +++ b/src/HOL/Inequalities.thy Sat Jul 18 22:58:50 2015 +0200 @@ -16,7 +16,7 @@ case (Suc i) have 0: "i = nat((n-1) - m)" "m \ n-1" using Suc(2,3) by arith+ have "\ {m..n} = \ {m..1+(n-1)}" by simp - also have "\ = \ {m..n-1} + n" using `m \ n` + also have "\ = \ {m..n-1} + n" using \m \ n\ by(subst atLeastAtMostPlus1_int_conv) simp_all also have "\ = ((n-1)*(n-1+1) - m*(m-1)) div 2 + n" by(simp add: Suc(1)[OF 0]) @@ -43,7 +43,7 @@ hence "{m..{m..{m..n-1}" by simp also have "\ = (n*(n-1) - m*(m-1)) div 2" - using assms `m < n` by (simp add: Setsum_Icc_nat mult.commute) + using assms \m < n\ by (simp add: Setsum_Icc_nat mult.commute) finally show ?thesis . next assume "\ m < n" with assms show ?thesis by simp