--- a/doc-src/TutorialI/Misc/arith4.thy Tue Sep 05 13:12:00 2000 +0200
+++ /dev/null Thu Jan 01 00:00:00 1970 +0000
@@ -1,8 +0,0 @@
-(*<*)
-theory arith4 = Main:;
-(*>*)
-lemma "\\<not> m < n \\<and> m < n+1 \\<Longrightarrow> m = n";
-(**)(*<*)
-by(arith);
-end
-(*>*)