aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Max.v
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-02-14 14:39:07 +0000
commit67f72c93f5f364591224a86c52727867e02a8f71 (patch)
treeecf630daf8346e77e6620233d8f3e6c18a0c9b3c /theories/Arith/Max.v
parentb239b208eb9a66037b0c629cf7ccb6e4b110636a (diff)
option -dump-glob pour coqdoc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2474 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Arith/Max.v')
-rwxr-xr-xtheories/Arith/Max.v11
1 files changed, 4 insertions, 7 deletions
diff --git a/theories/Arith/Max.v b/theories/Arith/Max.v
index 352bd236f..43c683a90 100755
--- a/theories/Arith/Max.v
+++ b/theories/Arith/Max.v
@@ -10,9 +10,7 @@
Require Arith.
-(**************************************************************************)
-(* maximum of two natural numbers *)
-(**************************************************************************)
+(** maximum of two natural numbers *)
Fixpoint max [n:nat] : nat -> nat :=
[m:nat]Cases n m of
@@ -21,8 +19,7 @@ Fixpoint max [n:nat] : nat -> nat :=
| (S n') (S m') => (S (max n' m'))
end.
-(* Simplifications of max *)
-
+(** Simplifications of [max] *)
Lemma max_SS : (n,m:nat)((S (max n m))=(max (S n) (S m))).
Proof.
@@ -34,7 +31,7 @@ Proof.
NewInduction n;NewInduction m;Simpl;Auto with arith.
Qed.
-(* max and le *)
+(** [max] and [le] *)
Lemma max_l : (n,m:nat)(le m n)->(max n m)=n.
Proof.
@@ -60,7 +57,7 @@ Qed.
Hints Resolve max_r max_l le_max_l le_max_r: arith v62.
-(* max n m is equal to n or m *)
+(** [max n m] is equal to [n] or [m] *)
Lemma max_dec : (n,m:nat){(max n m)=n}+{(max n m)=m}.
Proof.