summaryrefslogtreecommitdiff
path: root/test-suite/failure/clashes.v
blob: fcfd29fea6fd4012dfc55874888b26ddbf1e60c9 (plain)
1
2
3
4
5
6
7
8
(* Submitted by David Nowak *)

(* Simpler to forbid the definition of n as a global than to write it
   S.n to keep n accessible... *)

Section S.
Variable n:nat.
Inductive P : Set := n : P.