aboutsummaryrefslogtreecommitdiffstats
path: root/src/extraction/Extract.v
diff options
context:
space:
mode:
authorckeller <ckeller@users.noreply.github.com>2022-07-30 16:42:50 +0200
committerGitHub <noreply@github.com>2022-07-30 16:42:50 +0200
commitde9c46d059ddd38c0c1922d91cb788c3d550d488 (patch)
treedb0cdadd6853877cc02be40b325388f0a4d68a24 /src/extraction/Extract.v
parentd5697269991500ed1b4b3e6bbec6108ea3a059bb (diff)
downloadsmtcoq-de9c46d059ddd38c0c1922d91cb788c3d550d488.tar.gz
smtcoq-de9c46d059ddd38c0c1922d91cb788c3d550d488.zip
Extraction for Coq 8.13 (#109)
Extraction is back! Some new features: * Not only an executable is generated, but the ZChaff and veriT checkers are available through a package called Smtcoq_extr * The command-line arguments are better handled * The veriT checker is now the default
Diffstat (limited to 'src/extraction/Extract.v')
-rw-r--r--src/extraction/Extract.v9
1 files changed, 4 insertions, 5 deletions
diff --git a/src/extraction/Extract.v b/src/extraction/Extract.v
index 138a2ba..da484b5 100644
--- a/src/extraction/Extract.v
+++ b/src/extraction/Extract.v
@@ -10,13 +10,12 @@
(**************************************************************************)
-Require Int63Native.
-Require Import ExtractNative.
-Require Import SMTCoq.
+Add Rec LoadPath "." as SMTCoq.
-Extract Constant Int63Native.eqb => "fun i j -> ExtrNative.compare i j = ExtrNative.Eq".
+Require Import ExtrOCamlInt63.
+Require Import SMTCoq.
Set Extraction AccessOpaque.
Extraction "extraction/sat_checker.ml" Sat_Checker.checker.
-Extraction "extraction/smt_checker.ml" Euf_Checker.checker_ext.
+Extraction "extraction/smt_checker.ml" Checker_Ext.checker_ext.