add examples from Freek's top 100 theorems (thms 30, 73, 77)
(*<*)theory fakenat imports Main begin(*>*)text{*\noindentThe type \tydx{nat} of naturalnumbers is predefined to have the constructors \cdx{0} and~\cdx{Suc}.It behaves approximately as if it were declared like this:*}datatype nat = zero ("0") | Suc nat(*<*)end(*>*)