summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/3004.v
blob: 896b1958b04a9f337bf6f3720b456784448460af (plain)
1
2
3
4
5
6
7
Set Implicit Arguments.
Unset Strict Implicit.
Parameter (M : nat -> Type).
Parameter (mp : forall (T1 T2 : Type) (f : T1 -> T2), list T1 -> list T2).

Definition foo (s : list {n : nat & M n}) :=
  let exT := existT in mp (fun x => projT1 x) s.