aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-27 12:43:43 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-11-27 12:43:43 +0000
commit500fb40a37455123d888cc6a2b595319dcbe8d67 (patch)
tree172beacc0750d862095ca0fb150b3e36b16938d9 /theories
parent00150efde21b9e493a1578dc35a30025fc79d9d7 (diff)
Remettre une section dans fast_integer pour contourner un bug de définition locale
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@990 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories')
-rw-r--r--theories/Zarith/fast_integer.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/theories/Zarith/fast_integer.v b/theories/Zarith/fast_integer.v
index 93b574f96..aaf27e008 100644
--- a/theories/Zarith/fast_integer.v
+++ b/theories/Zarith/fast_integer.v
@@ -14,6 +14,8 @@ Require Plus.
Require Mult.
Require Minus.
+Section fast_integer.
+
Inductive positive : Set :=
xI : positive -> positive
| xO : positive -> positive
@@ -1439,3 +1441,5 @@ 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. \ No newline at end of file