aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Arith/Min.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/Min.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/Min.v')
-rwxr-xr-xtheories/Arith/Min.v10
1 files changed, 4 insertions, 6 deletions
diff --git a/theories/Arith/Min.v b/theories/Arith/Min.v
index 56d254c48..8a5de8703 100755
--- a/theories/Arith/Min.v
+++ b/theories/Arith/Min.v
@@ -10,9 +10,7 @@
Require Arith.
-(**************************************************************************)
-(* minimum of two natural numbers *)
-(**************************************************************************)
+(** minimum of two natural numbers *)
Fixpoint min [n:nat] : nat -> nat :=
[m:nat]Cases n m of
@@ -21,7 +19,7 @@ Fixpoint min [n:nat] : nat -> nat :=
| (S n') (S m') => (S (min n' m'))
end.
-(* Simplifications of min *)
+(** Simplifications of [min] *)
Lemma min_SS : (n,m:nat)((S (min n m))=(min (S n) (S m))).
Proof.
@@ -33,7 +31,7 @@ Proof.
NewInduction n;NewInduction m;Simpl;Auto with arith.
Qed.
-(* min and le *)
+(** [min] and [le] *)
Lemma min_l : (n,m:nat)(le n m)->(min n m)=n.
Proof.
@@ -58,7 +56,7 @@ NewInduction m; Simpl; Auto with arith.
Qed.
Hints Resolve min_l min_r le_min_l le_min_r : arith v62.
-(* min n m is equal to n or m *)
+(** [min n m] is equal to [n] or [m] *)
Lemma min_dec : (n,m:nat){(min n m)=n}+{(min n m)=m}.
Proof.