doc-src/TutorialI/Misc/natsum.thy
changeset 10171 59d6633835fa
parent 9834 109b11c4e77e
child 10538 d1bf9ca9008d
--- a/doc-src/TutorialI/Misc/natsum.thy	Mon Oct 09 09:33:45 2000 +0200
+++ b/doc-src/TutorialI/Misc/natsum.thy	Mon Oct 09 10:18:21 2000 +0200
@@ -17,7 +17,8 @@
 
 lemma "sum n + sum n = n*(Suc n)";
 apply(induct_tac n);
-by(auto);
+apply(auto);
+done
 
 (*<*)
 end