diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-09-15 18:19:27 +0200 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-09-15 18:19:27 +0200 |
commit | a14e7e107bde61ad72410d62802efd67dfe8c3e2 (patch) | |
tree | a0f6d6be75eff480f3c5b02d6eac2993996c5f45 | |
parent | 83ebacdb7f307451fc801637224c911eb0da9fea (diff) |
Fixing line break in test for #3559.
-rw-r--r-- | test-suite/bugs/closed/3559.v | 3 |
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). |