src/HOL/Tools/Sledgehammer/sledgehammer_prover_smt2.ML
changeset 57158 f028d93798e6
parent 57078 a91d126338a4
child 57159 24cbdebba35a
--- a/src/HOL/Tools/Sledgehammer/sledgehammer_prover_smt2.ML	Mon Jun 02 17:34:26 2014 +0200
+++ b/src/HOL/Tools/Sledgehammer/sledgehammer_prover_smt2.ML	Mon Jun 02 17:34:26 2014 +0200
@@ -85,8 +85,8 @@
    (139, Crashed)]
 val smt2_failures = z3_failures @ unix_failures
 
-fun failure_of_smt2_failure (SMT2_Failure.Counterexample {is_real_cex, ...}) =
-    if is_real_cex then Unprovable else GaveUp
+fun failure_of_smt2_failure (SMT2_Failure.Counterexample genuine) =
+    if genuine then Unprovable else GaveUp
   | failure_of_smt2_failure SMT2_Failure.Time_Out = TimedOut
   | failure_of_smt2_failure (SMT2_Failure.Abnormal_Termination code) =
     (case AList.lookup (op =) smt2_failures code of