doc-src/TutorialI/Misc/arith1.thy
changeset 10171 59d6633835fa
parent 9458 c613cd06d5cf
--- a/doc-src/TutorialI/Misc/arith1.thy	Mon Oct 09 09:33:45 2000 +0200
+++ b/doc-src/TutorialI/Misc/arith1.thy	Mon Oct 09 10:18:21 2000 +0200
@@ -1,7 +1,7 @@
 (*<*)
 theory arith1 = Main:;
 (*>*)
-lemma "\\<lbrakk> \\<not> m < n; m < n+1 \\<rbrakk> \\<Longrightarrow> m = n";
+lemma "\<lbrakk> \<not> m < n; m < n+1 \<rbrakk> \<Longrightarrow> m = n";
 (**)(*<*)
 by(auto);
 end