diff options
Diffstat (limited to 'test-suite/micromega/bug_11656.v')
| -rw-r--r-- | test-suite/micromega/bug_11656.v | 11 |
1 files changed, 11 insertions, 0 deletions
diff --git a/test-suite/micromega/bug_11656.v b/test-suite/micromega/bug_11656.v new file mode 100644 index 0000000000..19846ad50a --- /dev/null +++ b/test-suite/micromega/bug_11656.v @@ -0,0 +1,11 @@ +Require Import Lia. +Require Import NArith. +Open Scope N_scope. + +Goal forall (a b c: N), + a <> 0 -> + c <> 0 -> + a * ((b + 1) * c) <> 0. +Proof. + intros. nia. +Qed. |
