aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/4394.v
blob: 751f1e697d41995ae9ab9c108846462d93fdc2f6 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
(* -*- coq-prog-args: ("-emacs" "-compat" "8.4") -*- *)
Require Import Equality List.
Unset Strict Universe Declaration.
Inductive Foo I A := foo (B : Type) : A -> I B -> Foo I A.
Definition Family := Type -> Type.
Definition fooFamily family : Family := Foo family.
Inductive Empty {T} : T -> Prop := .
Theorem empty (family : Family) (a : fold_right prod unit (map (Foo family) nil)) (b : unit) :
  Empty (a, b) -> False.
Proof.
  intro e.
  dependent induction e.
Qed.