doc-src/Tutorial/Misc/NatSum.thy
author wenzelm
Wed, 20 Oct 1999 11:05:06 +0200
changeset 7886 8fa551e22e52
parent 5377 efb799c5ed3c
permissions -rw-r--r--
the settings environment is now statically scoped; tuned;

NatSum = Main +
consts sum :: nat => nat
primrec
"sum 0 = 0"
"sum (Suc n) = Suc n + sum n"
end