aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zquot.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/ZArith/Zquot.v')
-rw-r--r--theories/ZArith/Zquot.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zquot.v b/theories/ZArith/Zquot.v
index 9a95669f5..5b79fbce8 100644
--- a/theories/ZArith/Zquot.v
+++ b/theories/ZArith/Zquot.v
@@ -46,7 +46,7 @@ Qed.
has been chosen to be [a], so this equation holds even for [b=0].
*)
-Notation Z_quot_rem_eq := Z.quot_rem' (only parsing).
+Notation Z_quot_rem_eq := Z.quot_rem' (compat "8.3").
(** Then, the inequalities constraining the remainder:
The remainder is bounded by the divisor, in term of absolute values *)