aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Numbers/Natural
diff options
context:
space:
mode:
authorGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-28 16:27:28 +0000
committerGravatar pboutill <pboutill@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-09-28 16:27:28 +0000
commit56a2994e2ecc931836fb4ef8b2bdb027a705cfcd (patch)
tree14d0bb8cebf6e81059baf64b01ee0d03f8f6521a /theories/Numbers/Natural
parente09064ff153ee9f909e8c2c1ee2aaa249b324a78 (diff)
Minor fixes of 'make doc'
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13472 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Numbers/Natural')
-rw-r--r--theories/Numbers/Natural/BigN/NMake.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Numbers/Natural/BigN/NMake.v b/theories/Numbers/Natural/BigN/NMake.v
index d82e205a6..cea2e3195 100644
--- a/theories/Numbers/Natural/BigN/NMake.v
+++ b/theories/Numbers/Natural/BigN/NMake.v
@@ -273,7 +273,7 @@ Module Make (W0:CyclicType) <: NType.
lazy beta iota delta [iter_sym dom_op dom_t comparen_m]. reflexivity.
Qed.
-(** TODO: no need for ZnZ.Spec_rect , _ind, and so on... *)
+(** TODO: no need for ZnZ.Spec_rect , Spec_ind, and so on... *)
Theorem spec_compare : forall x y,
compare x y = Zcompare [x] [y].