aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/HoTT_coq_078.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/opened/HoTT_coq_078.v')
-rw-r--r--test-suite/bugs/opened/HoTT_coq_078.v2
1 files changed, 1 insertions, 1 deletions
diff --git a/test-suite/bugs/opened/HoTT_coq_078.v b/test-suite/bugs/opened/HoTT_coq_078.v
index a2c97d067..6c02cad56 100644
--- a/test-suite/bugs/opened/HoTT_coq_078.v
+++ b/test-suite/bugs/opened/HoTT_coq_078.v
@@ -35,7 +35,7 @@ Definition transport_prod' {A : Type} {P Q : A -> Type} {a a' : A} (p : a = a')
| idpath => idpath
end. (* success *)
-Fail Definition transport_prod {A : Type} {P Q : A -> Type} {a a' : A} (p : a = a')
+Definition transport_prod {A : Type} {P Q : A -> Type} {a a' : A} (p : a = a')
(z : P a * Q a)
: transport (fun a => P a * Q a) p z = (transport _ p (fst z), transport _ p (snd z))
:= match p with