From 8581e1a977518c354eb06820d3513238412af7de Mon Sep 17 00:00:00 2001 From: Hugo Herbelin Date: Mon, 30 Mar 2015 22:15:02 +0200 Subject: Accomodating #4166 (providing "Require Import OmegaTactic" as a replacement for 8.4's "Require Omega"). --- plugins/omega/Omega.v | 8 ++------ 1 file changed, 2 insertions(+), 6 deletions(-) (limited to 'plugins/omega/Omega.v') diff --git a/plugins/omega/Omega.v b/plugins/omega/Omega.v index 7400d4629..a5f90dd66 100644 --- a/plugins/omega/Omega.v +++ b/plugins/omega/Omega.v @@ -13,10 +13,11 @@ (* *) (**************************************************************************) -(* We do not require [ZArith] anymore, but only what's necessary for Omega *) +(* We import what is necessary for Omega *) Require Export ZArith_base. Require Export OmegaLemmas. Require Export PreOmega. + Declare ML Module "omega_plugin". Hint Resolve Z.le_refl Z.add_comm Z.add_assoc Z.mul_comm Z.mul_assoc Z.add_0_l @@ -25,11 +26,6 @@ Hint Resolve Z.le_refl Z.add_comm Z.add_assoc Z.mul_comm Z.mul_assoc Z.add_0_l Require Export Zhints. -(* -(* The constant minus is required in coq_omega.ml *) -Require Minus. -*) - Hint Extern 10 (_ = _ :>nat) => abstract omega: zarith. Hint Extern 10 (_ <= _) => abstract omega: zarith. Hint Extern 10 (_ < _) => abstract omega: zarith. -- cgit v1.2.3