doc-src/TutorialI/Misc/fakenat.thy
changeset 11418 53a402c10ba9
parent 9541 d17c0b34d5c8
child 16417 9bc16273c2d4
--- a/doc-src/TutorialI/Misc/fakenat.thy	Fri Jul 13 17:56:05 2001 +0200
+++ b/doc-src/TutorialI/Misc/fakenat.thy	Fri Jul 13 17:58:39 2001 +0200
@@ -3,8 +3,8 @@
 (*>*)
 
 text{*\noindent
-The type \isaindexbold{nat}\index{*0|bold}\index{*Suc|bold} of natural
-numbers is predefined and behaves like
+The type \tydx{nat} of natural
+numbers is predefined to have the constructors \cdx{0} and~\cdx{Suc}.  It  behaves as if it were declared like this:
 *}
 
 datatype nat = 0 | Suc nat