aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Raxioms.v
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-12 17:49:21 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-03-12 17:49:21 +0000
commitcb1ae314411d78952062e5092804b85d981ad6e1 (patch)
tree52b9a4058c89b5849d875a4c1129951f35e9c1b1 /theories/Reals/Raxioms.v
parent7cb6a61133b6e3c2cd5601282a1f472ff0104c1f (diff)
*** empty log message ***
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3761 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Raxioms.v')
-rw-r--r--theories/Reals/Raxioms.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/theories/Reals/Raxioms.v b/theories/Reals/Raxioms.v
index cda4273a5..455511633 100644
--- a/theories/Reals/Raxioms.v
+++ b/theories/Reals/Raxioms.v
@@ -15,6 +15,7 @@
Require Export ZArith_base.
Require Export Rsyntax.
Require Export TypeSyntax.
+Import R_scope.
(*********************************************************)
(* Field axioms *)
@@ -111,6 +112,8 @@ Fixpoint INR [n:nat]:R:=(Cases n of
|(S O) => ``1``
|(S n) => ``(INR n)+1``
end).
+Arguments Scope INR [nat_scope].
+
(**********************************************************)
(** Injection from [Z] to [R] *)
@@ -122,6 +125,7 @@ Definition IZR:Z->R:=[z:Z](Cases z of
|(POS n) => (INR (convert n))
|(NEG n) => ``-(INR (convert n))``
end).
+Arguments Scope IZR [Z_scope].
(**********************************************************)
(** [R] Archimedian *)