aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/QArith/Qcanon.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/Qcanon.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/Qcanon.v')
-rw-r--r--theories/QArith/Qcanon.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/theories/QArith/Qcanon.v b/theories/QArith/Qcanon.v
index bc87e05d3..026e850ea 100644
--- a/theories/QArith/Qcanon.v
+++ b/theories/QArith/Qcanon.v
@@ -9,6 +9,7 @@
(*i $Id$ i*)
Require Import QArith.
+Require Import Znumtheory.
Require Import Eqdep_dec.
(** [Qc] : A canonical representation of rational numbers.