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

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