| author | Thomas Lindae <thomas.lindae@in.tum.de> | 
| Wed, 17 Jul 2024 21:02:30 +0200 | |
| changeset 81077 | 664c1a6cc8c1 | 
| parent 80983 | 2cc651d3ce8e | 
| permissions | -rw-r--r-- | 
| 8745 | 1 | (*<*) | 
| 58860 | 2 | theory fakenat imports Main begin | 
| 8745 | 3 | (*>*) | 
| 4 | ||
| 67406 | 5 | text\<open>\noindent | 
| 11418 | 6 | The type \tydx{nat} of natural
 | 
| 56260 
3d79c132e657
modernized approximation, avoiding bad name binding;
 wenzelm parents: 
48985diff
changeset | 7 | numbers is predefined to have the constructors \cdx{0} and~\cdx{Suc}.
 | 
| 
3d79c132e657
modernized approximation, avoiding bad name binding;
 wenzelm parents: 
48985diff
changeset | 8 | It behaves approximately as if it were declared like this: | 
| 67406 | 9 | \<close> | 
| 8745 | 10 | |
| 80983 
2cc651d3ce8e
partial revert of d97fdabd9e2b, to build old documentation more reliably;
 wenzelm parents: 
80914diff
changeset | 11 | datatype nat = zero ("0") | Suc nat
 | 
| 8745 | 12 | (*<*) | 
| 13 | end | |
| 14 | (*>*) |