aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Zarith/fast_integer.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/Zarith/fast_integer.v')
-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