summaryrefslogtreecommitdiff
path: root/test-suite/output/Inductive.v
blob: 8ff91268a64a37236b693415fc520556f570c809 (plain)
1
2
3
4
5
6
7
Fail Inductive list' (A:Set) : Set :=
| nil' : list' A
| cons' : A -> list' A -> list' (A*A).

(* Check printing of let-ins *)
Inductive foo (A : Type) (x : A) (y := x) := Foo.
Print foo.