src/Doc/Tutorial/Misc/fakenat.thy
changeset 48985 5386df44a037
parent 16417 9bc16273c2d4
child 56260 3d79c132e657
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/src/Doc/Tutorial/Misc/fakenat.thy	Tue Aug 28 18:57:32 2012 +0200
@@ -0,0 +1,13 @@
+(*<*)
+theory fakenat imports Main begin;
+(*>*)
+
+text{*\noindent
+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
+(*<*)
+end
+(*>*)