aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zmisc.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-11 13:29:02 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-11 13:29:02 +0000
commit5cf454a285bfcead3c2f97c3669ef10bcb232df9 (patch)
tree7dc438ac28003452deec5ef01cf70d98e3908269 /theories/ZArith/Zmisc.v
parent26f0747a93e403b08a0432221a18591a91966eb0 (diff)
Conformité des commentaires au format coqweb
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1951 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/ZArith/Zmisc.v')
-rw-r--r--theories/ZArith/Zmisc.v10
1 files changed, 5 insertions, 5 deletions
diff --git a/theories/ZArith/Zmisc.v b/theories/ZArith/Zmisc.v
index 425baa53c..29ac55bb4 100644
--- a/theories/ZArith/Zmisc.v
+++ b/theories/ZArith/Zmisc.v
@@ -272,7 +272,7 @@ Save.
Hints Unfold Zeven Zodd : zarith.
-(* Zdiv2 is defined on all Z, but notice that for odd negative integers
+(* [Zdiv2] is defined on all [Z], but notice that for odd negative integers
* it is not the euclidean quotient: in that case we have n = 2*(n/2)-1
*)
@@ -380,7 +380,7 @@ Rewrite -> (Case (Zcompare_EGAL x y) of [h1,h2: ?]h2 end H0).
Assumption.
Save.
-(* Four very basic lemmas about Zle, Zlt, Zge, Zgt *)
+(* Four very basic lemmas about [Zle], [Zlt], [Zge], [Zgt] *)
Lemma Zle_Zcompare :
(x,y:Z)`x <= y` -> Case `x ?= y` of True True False end.
Intros x y; Unfold Zle; Elim `x ?=y`; Auto with arith.
@@ -401,7 +401,7 @@ Lemma Zgt_Zcompare :
Intros x y; Unfold Zgt; Elim `x ?= y`; Intros; Discriminate Orelse Trivial with arith.
Save.
-(* Lemmas about Zmin *)
+(* Lemmas about [Zmin] *)
Lemma Zmin_plus : (x,y,n:Z) `(Zmin (x+n)(y+n))=(Zmin x y)+n`.
Intros; Unfold Zmin.
@@ -411,7 +411,7 @@ Rewrite (Zcompare_Zplus_compatible x y n).
Case `x ?= y`; Apply Zplus_sym.
Save.
-(* Lemmas about absolu *)
+(* Lemmas about [absolu] *)
Lemma absolu_lt : (x,y:Z) `0 <= x < y` -> (lt (absolu x) (absolu y)).
Proof.
@@ -433,7 +433,7 @@ Compute. Intro H0. Discriminate H0. Intuition.
Intros. Absurd `0 <= (NEG p)`. Compute. Auto with arith. Intuition.
Save.
-(* Lemmas on Zle_bool used in contrib/graphs *)
+(* Lemmas on [Zle_bool] used in contrib/graphs *)
Lemma Zle_bool_imp_le : (x,y:Z) (Zle_bool x y)=true -> (Zle x y).
Proof.