src/HOL/NatArith.thy
changeset 14607 099575a938e5
parent 14208 144f45277d5a
child 14981 e73f8140af78
--- a/src/HOL/NatArith.thy	Fri Apr 16 21:00:07 2004 +0200
+++ b/src/HOL/NatArith.thy	Fri Apr 16 21:00:36 2004 +0200
@@ -33,12 +33,12 @@
 *}
 (* Careful: arith_tac produces counter examples!
 fun add_arith cs = cs addafter ("arith_tac", arith_tac);
-TODO: use arith_tac for force_tac in Provers/clasip.ML *)
+TODO: use arith_tac for force_tac in Provers/clasimp.ML *)
 
 lemmas [arith_split] = nat_diff_split split_min split_max
 
 
-subsubsection {* Generic summation indexed over natural numbers *}
+subsection {* Generic summation indexed over natural numbers *}
 
 consts
   Summation :: "(nat => 'a::{zero, plus}) => nat => 'a"