aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-20 08:41:10 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-20 08:41:10 +0000
commitb898ce8e51b7cf47ff0989453d20ef062a4c5454 (patch)
tree56651238f16e21b83a093c8b13321cb2f8659992 /theories
parent07d8a4440e6ce46d7d6aaf2d1a045e1c4d972c8a (diff)
Suppression de la section fast_integer qui cachait le nom du module éponyme
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@862 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Zarith/fast_integer.v3
1 files changed, 0 insertions, 3 deletions
diff --git a/theories/Zarith/fast_integer.v b/theories/Zarith/fast_integer.v
index 5d955f5ee..93b574f96 100644
--- a/theories/Zarith/fast_integer.v
+++ b/theories/Zarith/fast_integer.v
@@ -14,7 +14,6 @@ Require Plus.
Require Mult.
Require Minus.
-Section fast_integer.
Inductive positive : Set :=
xI : positive -> positive
| xO : positive -> positive
@@ -1440,5 +1439,3 @@ Intros x y;Case x;Case y; [
| Unfold Zcompare; Intros q p; Rewrite <- ZC4; Intros H; Exists (true_sub q p);
Simpl; Rewrite (ZC1 q p H); Trivial with arith].
Save.
-
-End fast_integer.