summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3792.v
blob: 39057b9c528be5050ad74ee70be94240f06e1e52 (plain)
1
2
3
4
Fail Definition pull_if_dep
: forall {A} (P : bool -> Type) (a : A true) (a' : A false)
         (b : bool),
    P (if b as b return A b then a else a').