aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/Reals/Ranalysis1.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-16 14:32:58 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-10-16 14:32:58 +0000
commitafe4da6f7d873471adaee010a5156ce6c117f8dc (patch)
tree04cdf3add27515131b0c6b1cc60c99a2fc5cae0d /theories/Reals/Ranalysis1.v
parentd7604922b69e2b3b0423dcec15dbdb9ae6993fdf (diff)
Pour eviter des regles redondantes en v7
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4647 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'theories/Reals/Ranalysis1.v')
-rw-r--r--theories/Reals/Ranalysis1.v14
1 files changed, 6 insertions, 8 deletions
diff --git a/theories/Reals/Ranalysis1.v b/theories/Reals/Ranalysis1.v
index 068b9367b..715b9a0ae 100644
--- a/theories/Reals/Ranalysis1.v
+++ b/theories/Reals/Ranalysis1.v
@@ -28,16 +28,14 @@ Definition div_real_fct [a:R;f:R->R] : R->R := [x:R] ``a/(f x)``.
Definition comp [f1,f2:R->R] : R->R := [x:R] ``(f1 (f2 x))``.
Definition inv_fct [f:R->R] : R->R := [x:R]``/(f x)``.
-Infix "+" plus_fct (at level 4, left associativity) : Rfun_scope.
-Notation "- x" := (opp_fct x) (at level 0) : Rfun_scope
- V8only (at level 40).
-Infix "*" mult_fct (at level 3, left associativity) : Rfun_scope.
-Infix "-" minus_fct (at level 4, left associativity) : Rfun_scope.
-Infix "/" div_fct (at level 3, left associativity) : Rfun_scope.
+V8Infix "+" plus_fct : Rfun_scope.
+V8Notation "- x" := (opp_fct x) : Rfun_scope.
+V8Infix "*" mult_fct : Rfun_scope.
+V8Infix "-" minus_fct : Rfun_scope.
+V8Infix "/" div_fct : Rfun_scope.
Notation Local "f1 'o' f2" := (comp f1 f2) (at level 2, right associativity)
: Rfun_scope.
-Notation "/ x" := (inv_fct x) (at level 0): Rfun_scope
- V8only (at level 30, left associativity).
+V8Notation "/ x" := (inv_fct x) : Rfun_scope.
Delimits Scope Rfun_scope with F.