aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/success
diff options
context:
space:
mode:
authorGravatar Maxime Dénès <mail@maximedenes.fr>2017-10-10 10:52:30 +0200
committerGravatar Maxime Dénès <mail@maximedenes.fr>2017-10-10 10:52:30 +0200
commita2e283c8545f9e7f2951c42892945b027674a665 (patch)
tree5fb5d5946a31f07b83f85eaa9206d9b586ee7b89 /test-suite/success
parent77eb48ff814ec92fdaf4c7b61026d642ac2f14a6 (diff)
parentee42eb1e10be8632e277cf8b9ac6ba40ef86372b (diff)
Merge PR #768: Omega and romega know about context definitions (fix old bug 148)
Diffstat (limited to 'test-suite/success')
-rw-r--r--test-suite/success/ROmega4.v26
1 files changed, 26 insertions, 0 deletions
diff --git a/test-suite/success/ROmega4.v b/test-suite/success/ROmega4.v
new file mode 100644
index 000000000..58ae5b8fb
--- /dev/null
+++ b/test-suite/success/ROmega4.v
@@ -0,0 +1,26 @@
+(** ROmega is now aware of the bodies of context variables
+ (of type Z or nat).
+ See also #148 for the corresponding improvement in Omega.
+*)
+
+Require Import ZArith ROmega.
+Open Scope Z.
+
+Goal let x := 3 in x = 3.
+intros.
+romega.
+Qed.
+
+(** Example seen in #4132
+ (actually solvable even if b isn't known to be 5) *)
+
+Lemma foo
+ (x y x' zxy zxy' z : Z)
+ (b := 5)
+ (Ry : - b <= y < b)
+ (Bx : x' <= b)
+ (H : - zxy' <= zxy)
+ (H' : zxy' <= x') : - b <= zxy.
+Proof.
+romega.
+Qed.