aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith/Qreduction.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-21 12:07:32 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-21 12:07:32 +0000
commit0a235f0d6ed807600ccf5534af7ed6f8657d1274 (patch)
tree2dfd27afd9386cb0e8c156dbd69e698bc0ff43ac /theories/QArith/Qreduction.v
parent0f4f723a5608075ff4aa48290314df30843efbcb (diff)
better scope/require managment (patch by Russel O'Connor)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9155 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/QArith/Qreduction.v')
-rw-r--r--theories/QArith/Qreduction.v5
1 files changed, 3 insertions, 2 deletions
diff --git a/theories/QArith/Qreduction.v b/theories/QArith/Qreduction.v
index 41e0d9a45..657a00ed5 100644
--- a/theories/QArith/Qreduction.v
+++ b/theories/QArith/Qreduction.v
@@ -11,7 +11,7 @@
(** * Normalisation functions for rational numbers. *)
Require Export QArith_base.
-Require Export Znumtheory.
+Require Import Znumtheory.
(** First, a function that (tries to) build a positive back from a Z. *)
@@ -60,6 +60,7 @@ assert (0 < dd).
rewrite <- H4; compute; auto.
rewrite Z2P_correct; auto.
ring.
+Close Scope Z_scope.
Qed.
Lemma Qred_complete : forall p q, p==q -> Qred p = Qred q.
@@ -132,7 +133,7 @@ intro H2; elim (Zmult_integral _ _ H2); auto.
replace (g'*g*(aa*dd)) with ((g*aa)*(g'*dd)); [|ring].
replace (g'*g*(bb*cc)) with ((g'*cc)*(g*bb)); [|ring].
rewrite <- Hg3; rewrite <- Hg4; rewrite <- Hg'3; rewrite <- Hg'4; auto.
-Open Scope Q_scope.
+Close Scope Z_scope.
Qed.
Add Morphism Qred : Qred_comp.