summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/HoTT_coq_012.v
blob: a3c697f8ca6fdb30faf9f40ed82b858ed600c6b8 (plain)
1
2
3
4
(* -*- mode: coq; coq-prog-args: ("-emacs" "-indices-matter") -*- *)

Definition UU := Type.
Inductive toto (B : UU) : UU := c (x : B).