diff options
| author | Pierre-Marie Pédrot | 2014-02-06 01:05:30 +0100 |
|---|---|---|
| committer | Pierre-Marie Pédrot | 2014-02-08 20:10:54 +0100 |
| commit | bd41c9d104550ad5472a28655cd6353ba6df1696 (patch) | |
| tree | 3dbe7fb15b4b32d7350fe87aca29f7e977dad5ab /plugins | |
| parent | 009fb68f0578e462b817f50772e2fba8d58c4f0d (diff) | |
Less dependencies in Omega.
Diffstat (limited to 'plugins')
| -rw-r--r-- | plugins/omega/Omega.v | 2 | ||||
| -rw-r--r-- | plugins/setoid_ring/InitialRing.v | 3 |
2 files changed, 2 insertions, 3 deletions
diff --git a/plugins/omega/Omega.v b/plugins/omega/Omega.v index ea5a8cb712..7e7b52bb90 100644 --- a/plugins/omega/Omega.v +++ b/plugins/omega/Omega.v @@ -54,4 +54,4 @@ Hint Extern 10 (~ (_ < _)%Z) => abstract omega: zarith. Hint Extern 10 (~ (_ >= _)%Z) => abstract omega: zarith. Hint Extern 10 (~ (_ > _)%Z) => abstract omega: zarith. -Hint Extern 10 False => abstract omega: zarith.
\ No newline at end of file +Hint Extern 10 False => abstract omega: zarith. diff --git a/plugins/setoid_ring/InitialRing.v b/plugins/setoid_ring/InitialRing.v index e805151ce4..ca178dd384 100644 --- a/plugins/setoid_ring/InitialRing.v +++ b/plugins/setoid_ring/InitialRing.v @@ -6,8 +6,7 @@ (* * GNU Lesser General Public License Version 2.1 *) (************************************************************************) -Require Import ZArith_base. -Require Import Zpow_def. +Require Import Zbool. Require Import BinInt. Require Import BinNat. Require Import Setoid. |
