diff options
Diffstat (limited to 'contrib/micromega/MExtraction.v')
-rw-r--r-- | contrib/micromega/MExtraction.v | 23 |
1 files changed, 0 insertions, 23 deletions
diff --git a/contrib/micromega/MExtraction.v b/contrib/micromega/MExtraction.v deleted file mode 100644 index a5ac92db..00000000 --- a/contrib/micromega/MExtraction.v +++ /dev/null @@ -1,23 +0,0 @@ -(************************************************************************) -(* v * The Coq Proof Assistant / The Coq Development Team *) -(* <O___,, * CNRS-Ecole Polytechnique-INRIA Futurs-Universite Paris Sud *) -(* \VV/ **************************************************************) -(* // * This file is distributed under the terms of the *) -(* * GNU Lesser General Public License Version 2.1 *) -(************************************************************************) -(* *) -(* Micromega: A reflexive tactic using the Positivstellensatz *) -(* *) -(* Frédéric Besson (Irisa/Inria) 2006-2008 *) -(* *) -(************************************************************************) - -(* Used to generate micromega.ml *) - -Require Import ZMicromega. -Require Import QMicromega. -Require Import VarMap. -Require Import RingMicromega. -Require Import NArith. - -Extraction "micromega.ml" List.map simpl_cone map_cone indexes n_of_Z Nnat.N_of_nat ZTautoChecker QTautoChecker find. |