aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zcomplements.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/ZArith/Zcomplements.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/ZArith/Zcomplements.v')
-rw-r--r--theories/ZArith/Zcomplements.v14
1 files changed, 8 insertions, 6 deletions
diff --git a/theories/ZArith/Zcomplements.v b/theories/ZArith/Zcomplements.v
index 5130c9807..ce9691450 100644
--- a/theories/ZArith/Zcomplements.v
+++ b/theories/ZArith/Zcomplements.v
@@ -12,8 +12,8 @@ Require ZArith.
Require Omega.
Require Wf_nat.
-(* Multiplication by a number >0 preserves Zcompare. It also perserves
- Zle, Zlt, Zge, Zgt *)
+(** Multiplication by a number >0 preserves [Zcompare]. It also perserves
+ [Zle], [Zlt], [Zge], [Zgt] *)
Implicit Arguments On.
@@ -174,9 +174,11 @@ Left ; Split with (NEG p); Reflexivity.
Right ; Split with `-1`; Reflexivity.
Save.
-(* The biggest power of 2 that is stricly less than a *)
-(* Easy to compute : replace all "1" of the binary representation by
- "0", except the first "1" (or the first one :-) *)
+(** The biggest power of 2 that is stricly less than [a]
+
+ Easy to compute: replace all "1" of the binary representation by
+ "0", except the first "1" (or the first one :-) *)
+
Fixpoint floor_pos [a : positive] : positive :=
Cases a of
| xH => xH
@@ -349,7 +351,7 @@ Save.
End diveucl.
-(* Two more induction principles upon Z. *)
+(** Two more induction principles over [Z]. *)
Theorem Z_lt_abs_rec : (P: Z -> Set)
((n: Z) ((m: Z) `|m|<|n|` -> (P m)) -> (P n)) -> (p: Z) (P p).