aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Raxioms.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-16 16:56:11 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-04-16 16:56:11 +0000
commite94f8b40f52e3c25c431082af80fc522cdfa098d (patch)
treeb31fc40e230247509fce5916db7432d74cc5c629 /theories/Reals/Raxioms.v
parent7d9eb40cad437c9a6bfe7eea588ca56cc50ed3ed (diff)
sumboolT, sumorT, sigTT, SigT redondants
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@3927 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Raxioms.v')
-rw-r--r--theories/Reals/Raxioms.v15
1 files changed, 15 insertions, 0 deletions
diff --git a/theories/Reals/Raxioms.v b/theories/Reals/Raxioms.v
index 64671d00d..e90fa2148 100644
--- a/theories/Reals/Raxioms.v
+++ b/theories/Reals/Raxioms.v
@@ -17,6 +17,21 @@ Require Export Rsyntax.
Require Export TypeSyntax.
V7only [Import R_scope.]. Open Local Scope R_scope.
+V7only [
+(*********************************************************)
+(* Compatibility *)
+(*********************************************************)
+Notation sumboolT := Specif.sumbool.
+Notation leftT := Specif.left.
+Notation rightT := Specif.right.
+Notation sumorT := Specif.sumor.
+Notation inleftT := Specif.inleft.
+Notation inrightT := Specif.inright.
+Notation sigTT := Specif.sigT.
+Notation existTT := Specif.existT.
+Notation SigT := Specif.sigT.
+].
+
(*********************************************************)
(* Field axioms *)
(*********************************************************)