src/HOL/Set_Interval.thy
changeset 56480 093ea91498e6
parent 56328 b3551501424e
child 56949 d1a937cbf858
--- a/src/HOL/Set_Interval.thy	Wed Apr 09 09:37:47 2014 +0200
+++ b/src/HOL/Set_Interval.thy	Wed Apr 09 09:37:48 2014 +0200
@@ -1594,13 +1594,7 @@
 proof -
   from assms obtain y where "y = x - 1" and "y \<noteq> 0" by simp_all
   moreover have "(\<Sum>i<n. (y + 1) ^ i) = ((y + 1) ^ n - 1) / y"
-  proof (induct n)
-    case 0 then show ?case by simp
-  next
-    case (Suc n)
-    moreover from Suc `y \<noteq> 0` have "(1 + y) ^ n = (y * inverse y) * (1 + y) ^ n" by simp 
-    ultimately show ?case by (simp add: field_simps divide_inverse)
-  qed
+    by (induct n) (simp_all add: field_simps `y \<noteq> 0`)
   ultimately show ?thesis by simp
 qed