doc-src/TutorialI/Misc/fakenat.thy
changeset 9541 d17c0b34d5c8
parent 9494 44fefb6e9994
child 11418 53a402c10ba9
--- a/doc-src/TutorialI/Misc/fakenat.thy	Fri Aug 04 23:02:11 2000 +0200
+++ b/doc-src/TutorialI/Misc/fakenat.thy	Sun Aug 06 15:26:53 2000 +0200
@@ -7,7 +7,7 @@
 numbers is predefined and behaves like
 *}
 
-datatype nat = "0" | Suc nat
+datatype nat = 0 | Suc nat
 (*<*)
 end
 (*>*)