diff options
| author | Vincent Laporte | 2021-04-14 15:20:43 +0200 |
|---|---|---|
| committer | Vincent Laporte | 2021-04-14 15:20:43 +0200 |
| commit | 90a6c01dec9d58fa409e7097ac5ba03f08a9ae7b (patch) | |
| tree | 77260cc386ae0eafcbfec1d2a862f9e721e56b34 /test-suite/micromega/example.v | |
| parent | ea62d1e19f2ba565ea3a18ba3709a06af5c845ac (diff) | |
| parent | 8193ca191cc435c108a4842ae38a11d74c7c20a5 (diff) | |
Merge PR #14045: Zify: more aggressive application of saturation rules
Reviewed-by: vbgl
Diffstat (limited to 'test-suite/micromega/example.v')
| -rw-r--r-- | test-suite/micromega/example.v | 6 |
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/micromega/example.v b/test-suite/micromega/example.v index d70bb809c6..d22e2b7c8c 100644 --- a/test-suite/micromega/example.v +++ b/test-suite/micromega/example.v @@ -12,6 +12,12 @@ Open Scope Z_scope. Require Import ZMicromega. Require Import VarMap. +Lemma power_pos : forall x y, 0 <= x \/ False -> x^ y >= 0. +Proof. + intros. + lia. +Qed. + Lemma not_so_easy : forall x n : Z, 2*x + 1 <= 2 *n -> x <= n-1. Proof. |
