aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssreflect/eqtype.v
diff options
context:
space:
mode:
authorEnrico Tassi2018-09-03 15:02:21 +0200
committerEnrico Tassi2018-09-04 15:10:48 +0200
commit360a8819a08c4cf005d96f0ac6bff65903dccfd4 (patch)
treebb48bc66c8ff0e65be1426c3660c923034480e9b /mathcomp/ssreflect/eqtype.v
parent1dcea6744ecc79546905d41a23801b1fc7b60c5a (diff)
[warnings] -w "+compatibility-notation" clean
Diffstat (limited to 'mathcomp/ssreflect/eqtype.v')
-rw-r--r--mathcomp/ssreflect/eqtype.v6
1 files changed, 3 insertions, 3 deletions
diff --git a/mathcomp/ssreflect/eqtype.v b/mathcomp/ssreflect/eqtype.v
index 01ce7a9..7721f0e 100644
--- a/mathcomp/ssreflect/eqtype.v
+++ b/mathcomp/ssreflect/eqtype.v
@@ -784,9 +784,9 @@ Canonical option_eqType := Eval hnf in EqType (option T) option_eqMixin.
End OptionEqType.
-Definition tag := projS1.
-Definition tagged I T_ : forall u, T_(tag u) := @projS2 I [eta T_].
-Definition Tagged I i T_ x := @existS I [eta T_] i x.
+Definition tag := projT1.
+Definition tagged I T_ : forall u, T_(tag u) := @projT2 I [eta T_].
+Definition Tagged I i T_ x := @existT I [eta T_] i x.
Arguments Tagged [I i].
Prenex Implicits tag tagged Tagged.