aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-24 13:04:02 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2006-10-24 13:04:02 +0000
commit23811536c3e85865ceb70136c8a3403d7f6f0c48 (patch)
treea2b6e0aa23de6e645c5b74a3d9d49791f2cacf57
parent2ea9a0b938edb872eb2f7bbaabc05ba8ed39295e (diff)
Test apply in
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@9270 85f007b7-540e-0410-9357-904b9bb8a0f7
-rw-r--r--test-suite/success/apply.v14
1 files changed, 14 insertions, 0 deletions
diff --git a/test-suite/success/apply.v b/test-suite/success/apply.v
new file mode 100644
index 000000000..4f2606963
--- /dev/null
+++ b/test-suite/success/apply.v
@@ -0,0 +1,14 @@
+(* Test apply in *)
+
+Goal (forall x y, x = S y -> y=y) -> 2 = 4 -> 3=3.
+intros H H0.
+apply H in H0.
+assumption.
+Qed.
+
+Require Import ZArith.
+Open Scope Z_scope.
+Goal forall x y z, ~ z <= 0 -> x * z < y * z -> x <= y.
+intros; apply Znot_le_gt, Zgt_lt in H.
+apply Zmult_lt_reg_r, Zlt_le_weak in H0; auto.
+Qed.