summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/shouldsucceed/2307.v
blob: 7c04949539f870d926eb35d34e9c28e094417b37 (plain)
1
2
3
Inductive V: nat -> Type := VS n: V (S n).
Definition f (e: V 1): nat := match e with VS 0 => 3 end.