aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/eqtype.v
diff options
context:
space:
mode:
authorMaxime Dénès2017-10-30 14:16:48 +0100
committerMaxime Dénès2017-10-30 14:16:48 +0100
commite1b1743fb6aaed042d5e6762ea76c3242593ab1d (patch)
treef2c7a9504fe1a1a39a9015a771bf07eba1696ca8 /mathcomp/ssreflect/eqtype.v
parentd5437703555329168288467dc1a94b1176e1776e (diff)
Fix obsolete vernacular syntax for locality.
It was emitting a deprecation warning and will soon be removed from Coq.
Diffstat (limited to 'mathcomp/ssreflect/eqtype.v')
-rw-r--r--mathcomp/ssreflect/eqtype.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/mathcomp/ssreflect/eqtype.v b/mathcomp/ssreflect/eqtype.v
index e11fd9f..3e8230e 100644
--- a/mathcomp/ssreflect/eqtype.v
+++ b/mathcomp/ssreflect/eqtype.v
@@ -696,7 +696,7 @@ Section SubEqType.
Variables (T : eqType) (P : pred T) (sT : subType P).
-Notation Local ev_ax := (fun T v => @Equality.axiom T (fun x y => v x == v y)).
+Local Notation ev_ax := (fun T v => @Equality.axiom T (fun x y => v x == v y)).
Lemma val_eqP : ev_ax sT val. Proof. exact: inj_eqAxiom val_inj. Qed.
Definition sub_eqMixin := EqMixin val_eqP.