aboutsummaryrefslogtreecommitdiffhomepage
path: root/theories/ZArith/Zmin.v
diff options
context:
space:
mode:
Diffstat (limited to 'theories/ZArith/Zmin.v')
-rw-r--r--theories/ZArith/Zmin.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/theories/ZArith/Zmin.v b/theories/ZArith/Zmin.v
index 2c5003a6d..fbb31632c 100644
--- a/theories/ZArith/Zmin.v
+++ b/theories/ZArith/Zmin.v
@@ -45,7 +45,7 @@ Proof Z.min_le_compat_l.
(** * Semi-lattice properties of min *)
Lemma Zmin_idempotent : forall n, Z.min n n = n. Proof Z.min_id.
-Notation Zmin_n_n := Z.min_id (only parsing).
+Notation Zmin_n_n := Z.min_id (compat "8.3").
Lemma Zmin_comm : forall n m, Z.min n m = Z.min m n. Proof Z.min_comm.
Lemma Zmin_assoc : forall n m p, Z.min n (Z.min m p) = Z.min (Z.min n m) p.
Proof Z.min_assoc.