aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/ArithProp.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-26 12:13:06 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-09-26 12:13:06 +0000
commit4aec8fda1161953cf929b4e282eea9b672ab4058 (patch)
treeeea4b8ab24fdea8fb05206b1764ce1ed3c752d72 /theories/Reals/ArithProp.v
parent351a500eada776832ac9b09657e42f5d6cd7210f (diff)
commit de field + renommages
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9179 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/ArithProp.v')
-rw-r--r--theories/Reals/ArithProp.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/Reals/ArithProp.v b/theories/Reals/ArithProp.v
index c05ea465d..a00d42879 100644
--- a/theories/Reals/ArithProp.v
+++ b/theories/Reals/ArithProp.v
@@ -12,7 +12,7 @@ Require Import Rbase.
Require Import Rbasic_fun.
Require Import Even.
Require Import Div2.
-Require Import NewArithRing.
+Require Import ArithRing.
Open Local Scope Z_scope.
Open Local Scope R_scope.