aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/inds_type_sec.v
blob: af31940db6438ab0888f2c5040e00d9ce6409a00 (plain)
1
2
3
Section S.
Inductive T [U:Type] : Set := c : U -> (T U).
End S.