aboutsummaryrefslogtreecommitdiffhomepage
path: root/contrib/ring/Ring_theory.v
diff options
context:
space:
mode:
Diffstat (limited to 'contrib/ring/Ring_theory.v')
-rw-r--r--contrib/ring/Ring_theory.v15
1 files changed, 10 insertions, 5 deletions
diff --git a/contrib/ring/Ring_theory.v b/contrib/ring/Ring_theory.v
index 1c48c4b45..08bb53955 100644
--- a/contrib/ring/Ring_theory.v
+++ b/contrib/ring/Ring_theory.v
@@ -25,8 +25,8 @@ Variable Azero : A.
is a good choice. The proof of A_eq_prop is in this case easy. *)
Variable Aeq : A -> A -> bool.
-Infix 4 "+" Aplus.
-Infix 4 "*" Amult.
+Infix 4 "+" Aplus V8only 40 (left associativity).
+Infix 4 "*" Amult V8only 30 (left associativity).
Notation "0" := Azero.
Notation "1" := Aone.
@@ -146,11 +146,16 @@ Variable Azero : A.
Variable Aopp : A -> A.
Variable Aeq : A -> A -> bool.
-Infix 4 "+" Aplus.
-Infix 4 "*" Amult.
+Infix 4 "+" Aplus V8only 40 (left associativity).
+Infix 4 "*" Amult V8only 30 (left associativity).
Notation "0" := Azero.
Notation "1" := Aone.
-Notation "- x" := (Aopp x) (at level 3).
+Notation "- 0" := (Aopp Azero) (at level 3)
+ V8only (at level 40, left associativity).
+Notation "- 1" := (Aopp Aone) (at level 3)
+ V8only (at level 40, left associativity).
+Notation "- x" := (Aopp x) (at level 3)
+ V8only (at level 40, left associativity).
Record Ring_Theory : Prop :=
{ Th_plus_sym : (n,m:A) n + m == m + n;