aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/failure/clashes.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-04-12 12:55:01 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2002-04-12 12:55:01 +0000
commitb1f64fc34b3d845571830970cf8c8ff0f6525530 (patch)
tree5631c56af82669e6bfc55a84da0b84651c8dcb30 /test-suite/failure/clashes.v
parent890696ca0c475a8e169882c49256356cd96b447f (diff)
*** empty log message ***
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2638 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/failure/clashes.v')
-rw-r--r--test-suite/failure/clashes.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/failure/clashes.v b/test-suite/failure/clashes.v
new file mode 100644
index 000000000..fcfd29fea
--- /dev/null
+++ b/test-suite/failure/clashes.v
@@ -0,0 +1,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.