updated SMT2 examples and certificates
authorblanchet
Thu, 13 Mar 2014 16:21:09 +0100
changeset 56112 040424c3800d
parent 56111 5b76e1790c38
child 56115 9bf84c452463
updated SMT2 examples and certificates
src/HOL/SMT_Examples/SMT_Tests.thy
src/HOL/Tools/SMT2/smt2_solver.ML
--- a/src/HOL/SMT_Examples/SMT_Tests.thy	Thu Mar 13 16:17:14 2014 +0100
+++ b/src/HOL/SMT_Examples/SMT_Tests.thy	Thu Mar 13 16:21:09 2014 +0100
@@ -127,7 +127,7 @@
   "\<exists>x. P x \<longrightarrow> P a \<and> P b"
   "\<exists>x. (\<exists>y. P y) \<longrightarrow> P x"
   "(\<exists>x. Q \<longrightarrow> P x) \<longleftrightarrow> (Q \<longrightarrow> (\<exists>x. P x))"
-  by smt2+
+  oops (* smt2 FIXME: requires Z3 4.3.1 *)
 
 lemma
   "(\<not>(\<exists>x. P x)) \<longleftrightarrow> (\<forall>x. \<not> P x)"
@@ -146,7 +146,7 @@
   "(\<exists>x. \<forall>y. P x \<longleftrightarrow> P y) \<longrightarrow> ((\<exists>x. P x) \<longleftrightarrow> (\<forall>y. P y))"
   "\<exists>z. P z \<longrightarrow> (\<forall>x. P x)"
   "(\<exists>y. \<forall>x. R x y) \<longrightarrow> (\<forall>x. \<exists>y. R x y)"
-  by smt2+
+  by smt+ (* smt2 FIXME: requires Z3 4.3.1 *)
 
 lemma
   "(\<exists>!x. P x) \<longrightarrow> (\<exists>x. P x)"
--- a/src/HOL/Tools/SMT2/smt2_solver.ML	Thu Mar 13 16:17:14 2014 +0100
+++ b/src/HOL/Tools/SMT2/smt2_solver.ML	Thu Mar 13 16:21:09 2014 +0100
@@ -124,7 +124,7 @@
   let
     val options = SMT2_Config.solver_options_of ctxt
     val cmd = command ()
-    val comments = [space_implode " " (cmd @ options)]
+    val comments = [space_implode " " options]
 
     val (str, replay_data as {context=ctxt', ...}) =
       ithms