aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3559.v
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-09-15 18:19:27 +0200
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-09-15 18:19:27 +0200
commita14e7e107bde61ad72410d62802efd67dfe8c3e2 (patch)
treea0f6d6be75eff480f3c5b02d6eac2993996c5f45 /test-suite/bugs/closed/3559.v
parent83ebacdb7f307451fc801637224c911eb0da9fea (diff)
Fixing line break in test for #3559.
Diffstat (limited to 'test-suite/bugs/closed/3559.v')
-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).