src/HOL/Isar_examples/Summation.thy
changeset 9659 b9cf6801f3da
parent 8814 0a5edcbe0695
child 10007 64bf7da1994a
--- a/src/HOL/Isar_examples/Summation.thy	Sat Aug 19 12:44:20 2000 +0200
+++ b/src/HOL/Isar_examples/Summation.thy	Sat Aug 19 12:44:39 2000 +0200
@@ -153,7 +153,8 @@
   show "?P 0"; by (simp add: power_eq_if);
 
   fix n;
-  have "?S (n + 1) = ?S n + #4 * (n + 1)^#3"; by (simp add: power_eq_if distrib);
+  have "?S (n + 1) = ?S n + #4 * (n + 1)^#3";
+    by (simp add: power_eq_if distrib);
   also; assume "?S n = (n * (n + 1))^2";
   also; have "... + #4 * (n + 1)^#3 = ((n + 1) * ((n + 1) + 1))^2";
     by (simp add: power_eq_if distrib);