doc-src/TutorialI/Misc/arith3.thy
changeset 8745 13b32661dde4
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/doc-src/TutorialI/Misc/arith3.thy	Wed Apr 19 11:56:31 2000 +0200
@@ -0,0 +1,8 @@
+(*<*)
+theory arith3 = Main:;
+(*>*)
+lemma "n*n = n \\<Longrightarrow> n=0 \\<or> n=1";
+(**)(*<*)
+oops;
+end
+(*>*)