new toplevel commands `Goal' and `Goalw';
isatool fixgoal;
(* Title: HOL/ex/natsum.thy ID: $Id$ Author: Tobias Nipkow Copyright 1994 TU MuenchenA summation operator. sum(f,n+1) is the sum of all f(i), i=0...n.*)NatSum = Arith +consts sum :: [nat=>nat, nat] => natprimrec "sum" nat "sum f 0 = 0" "sum f (Suc n) = f(n) + sum f n"end