summaryrefslogtreecommitdiff
path: root/test-suite/failure/Case14.v
blob: ba0c51a1526b71606fe9d092727116e8e26d018e (plain)
1
2
3
4
5
6
7
8
9
Inductive List (A : Set) : Set :=
  | Nil : List A
  | Cons : A -> List A -> List A.

Definition NIL := Nil nat.
Type match Nil nat return (List nat) with
     | NIL => NIL
     | _ => NIL
     end.