aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/failure/inductive1.v
blob: 7f42e7e16414454c006f264d09a04e2681586716 (plain)
1
2
3
4
(* A check that sort-polymorphic product is not set too low *)

Inductive prod (A B:Type) : Type := pair : A -> B -> prod A B.
Fail Check (fun (A:Type) (B:Prop) => (prod A B : Prop)).