aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success/Hints.v
diff options
context:
space:
mode:
authorGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-21 18:05:41 +0000
committerGravatar letouzey <letouzey@85f007b7-540e-0410-9357-904b9bb8a0f7>2011-02-21 18:05:41 +0000
commit5d9d019b1978f1a3ebb8429fcf23d8da9bf52212 (patch)
tree036fc4e6de72614a641c38adfa1104fa78dc3c7f /test-suite/success/Hints.v
parent440af48253bb8b9870c78e1392f0c7a10c23feee (diff)
Some fixes of the test-suite scripts
In particular, the Fail meta-command cannot for the moment catch a Syntax Error, which is raised by Vernac.parse_sentence, before we even now that the line starts by a Fail... git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13847 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/success/Hints.v')
-rw-r--r--test-suite/success/Hints.v4
1 files changed, 3 insertions, 1 deletions
diff --git a/test-suite/success/Hints.v b/test-suite/success/Hints.v
index 4aa00e689..6bbb0ff17 100644
--- a/test-suite/success/Hints.v
+++ b/test-suite/success/Hints.v
@@ -24,7 +24,7 @@ Hint Destruct h8 := 4 Hypothesis (_ <= _) => fun H => apply H.
(* Checks that local names are accepted *)
Section A.
Remark Refl : forall (A : Set) (x : A), x = x.
- Proof. exact refl_equal. Defined.
+ Proof. exact @refl_equal. Defined.
Definition Sym := sym_equal.
Let Trans := trans_equal.
@@ -51,6 +51,8 @@ Axiom a : forall n, n=0 <-> n<=0.
Hint Resolve -> a.
Goal forall n, n=0 -> n<=0.
auto.
+
+Print Hints
Qed.