blob: 207d62b956ef9627414ad095d966ba81fdcc7d78 (
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.
Inductive P : Set :=
n : P.
|