summaryrefslogtreecommitdiff
path: root/test-suite/success/apply.v
blob: 4f26069633c087e9248814b618bb5f06393c66c9 (plain)
1
2
3
4
5
6
7
8
9
10
11
12
13
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.