summaryrefslogtreecommitdiff
path: root/test-suite/failure/clashes.v
blob: 1a59ec66d13538ca7521b7beaa86a20798588035 (plain)
1
2
3
4
5
6
7
8
9
(* 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.
Fail Inductive P : Set :=
    n : P.