aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--test-suite/bugs/closed/3559.v3
1 files changed, 1 insertions, 2 deletions
diff --git a/test-suite/bugs/closed/3559.v b/test-suite/bugs/closed/3559.v
index 66d653c52..50645090f 100644
--- a/test-suite/bugs/closed/3559.v
+++ b/test-suite/bugs/closed/3559.v
@@ -18,8 +18,7 @@ Open Scope type_scope.
Definition iff A B := prod (A -> B) (B -> A).
Infix "<->" := iff : type_scope.
-Inductive paths {A : Type@{i}} (a : A) : A -> Type@{i} := idpath : paths a a where "x =
-y" := (@paths _ x y) : type_scope.
+Inductive paths {A : Type@{i}} (a : A) : A -> Type@{i} := idpath : paths a a where "x = y" := (@paths _ x y) : type_scope.
Class Contr_internal (A : Type) := { center : A ; contr : (forall y : A, center
= y) }.
Inductive trunc_index : Type := minus_two | trunc_S (_ : trunc_index).