doc-src/TutorialI/Misc/natsum.thy
author kleing
Wed, 12 Jul 2000 14:47:55 +0200
changeset 9287 c406d0af9368
parent 8745 13b32661dde4
child 9458 c613cd06d5cf
permissions -rw-r--r--
about.html -> logics.html

(*<*)
theory natsum = Main:;
(*>*)
text{*\noindent
In particular, there are \isa{case}-expressions, for example
*}

(*<*)term(*>*) "case n of 0 \\<Rightarrow> 0 | Suc m \\<Rightarrow> m";

text{*\noindent
primitive recursion, for example
*}

consts sum :: "nat \\<Rightarrow> nat";
primrec "sum 0 = 0"
        "sum (Suc n) = Suc n + sum n";

text{*\noindent
and induction, for example
*}

lemma "sum n + sum n = n*(Suc n)";
apply(induct_tac n);
apply(auto).;

(*<*)
end
(*>*)