tuned comments;
authorwenzelm
Tue, 05 Jun 2007 16:26:06 +0200
changeset 23253 b1f3f53c60b5
parent 23252 67268bb40b21
child 23254 99644a53f16d
tuned comments;
src/HOL/Presburger.thy
src/HOL/Tools/Presburger/cooper_dec.ML
src/HOL/ex/Abstract_NAT.thy
--- a/src/HOL/Presburger.thy	Tue Jun 05 16:26:04 2007 +0200
+++ b/src/HOL/Presburger.thy	Tue Jun 05 16:26:06 2007 +0200
@@ -1,9 +1,6 @@
 (*  Title:      HOL/Presburger.thy
     ID:         $Id$
     Author:     Amine Chaieb, Tobias Nipkow and Stefan Berghofer, TU Muenchen
-
-File containing necessary theorems for the proof
-generation for Cooper Algorithm  
 *)
 
 header {* Presburger Arithmetic: Cooper's Algorithm *}
--- a/src/HOL/Tools/Presburger/cooper_dec.ML	Tue Jun 05 16:26:04 2007 +0200
+++ b/src/HOL/Tools/Presburger/cooper_dec.ML	Tue Jun 05 16:26:06 2007 +0200
@@ -2,10 +2,8 @@
     ID:         $Id$
     Author:     Amine Chaieb and Tobias Nipkow, TU Muenchen
 
-File containing the implementation of Cooper Algorithm
-decision procedure (intensively inspired from J.Harrison)
-*)
-
+The Cooper Algorithm decision procedure (intensively inspired by
+J. Harrison). *)
 
 signature COOPER_DEC = 
 sig
--- a/src/HOL/ex/Abstract_NAT.thy	Tue Jun 05 16:26:04 2007 +0200
+++ b/src/HOL/ex/Abstract_NAT.thy	Tue Jun 05 16:26:06 2007 +0200
@@ -3,7 +3,7 @@
     Author:     Makarius
 *)
 
-header {* Abstract Natural Numbers with polymorphic recursion *}
+header {* Abstract Natural Numbers primitive recursion *}
 
 theory Abstract_NAT
 imports Main