summaryrefslogtreecommitdiff
path: root/test-suite/bugs/opened/shouldnotfail/743.v
blob: f1eee6c188c5f7bc0930e5a4079d0bf9132b04bb (plain)
1
2
3
4
5
6
7
8
9
10
11
12
Require Import Omega.

Lemma foo : forall n m : Z, (n >= 0)%Z -> (n * m >= 0)%Z -> (n <= n + n * m)%Z.
Proof.
  intros. omega.
Qed.

Lemma foo' : forall n m : nat, n <=  n + n * m.
Proof.
  intros. omega.
Qed.