disable triviality checking -- it might be the source of the spurious Interrupt exceptions that make it almost impossible to run Judgement Day
authorblanchet
Tue, 23 Nov 2010 23:10:13 +0100
changeset 40670 c059d550afec
parent 40669 5c316d1327d4
child 40676 23904fa13e03
child 40677 f5caf58e9cdb
disable triviality checking -- it might be the source of the spurious Interrupt exceptions that make it almost impossible to run Judgement Day
src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML
--- a/src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML	Tue Nov 23 22:37:16 2010 +0100
+++ b/src/HOL/Mirabelle/Tools/mirabelle_sledgehammer.ML	Tue Nov 23 23:10:13 2010 +0100
@@ -526,9 +526,12 @@
       val (prover_name, _) = get_prover ctxt args
       val minimize = AList.defined (op =) args minimizeK
       val metis_ft = AList.defined (op =) args metis_ftK
-      val trivial = TimeLimit.timeLimit try_outer_timeout
+      val trivial = false
+(* FIXME
+       TimeLimit.timeLimit try_outer_timeout
                                    (Try.invoke_try (SOME try_inner_timeout)) pre
                     handle TimeLimit.TimeOut => false
+*)
       fun apply_reconstructor m1 m2 =
         if metis_ft
         then