summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/2775.v
blob: f1f384bdf77433a0aab83f4b023ffe417dbf9ab5 (plain)
1
2
3
4
5
6
Inductive typ : forall (T:Type), list T ->  Type -> Prop :=
  | Get : forall (T:Type) (l:list T), typ T l T.


Derive Inversion inv with 
(forall (X: Type) (y: list nat), typ nat y X)  Sort Prop.