aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/ProgramWf.v
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-11-30 10:36:22 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-11-30 10:36:22 +0000
commit6bee8342c0a914376688fba3927352f826aa9942 (patch)
tree9bb6bd70ca7b0841806daf9b8a17840a8d3bd4fe /test-suite/success/ProgramWf.v
parentb7033be417da7b84a2fe723e02bf3c4efc55e6b0 (diff)
Quick hack to avoid anomaly on using Program w/o having required JMeq.
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@14749 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/ProgramWf.v')
-rw-r--r--test-suite/success/ProgramWf.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/success/ProgramWf.v b/test-suite/success/ProgramWf.v
index 81bdbc29f..00a13aed0 100644
--- a/test-suite/success/ProgramWf.v
+++ b/test-suite/success/ProgramWf.v
@@ -1,3 +1,9 @@
+(* Before loading Program, check non-anomaly on missing library Program *)
+
+Fail Program Definition f n (e:n=n): {n|n=0} := match n,e with 0, refl => 0 | _, _ => 0 end.
+
+(* Then we test Program properly speaking *)
+
Require Import Arith Program.
Require Import ZArith Zwf.