src/HOL/Mirabelle/Tools/mirabelle.ML
changeset 39377 9e544eb396dc
parent 39232 69c6d3e87660
child 39451 8893562a954b
equal deleted inserted replaced
39376:ca81b7ae543c 39377:9e544eb396dc
   158   let
   158   let
   159     val {context = ctxt, facts, goal} = Proof.goal st
   159     val {context = ctxt, facts, goal} = Proof.goal st
   160     val full_tac = HEADGOAL (Method.insert_tac facts THEN' tac ctxt)
   160     val full_tac = HEADGOAL (Method.insert_tac facts THEN' tac ctxt)
   161   in
   161   in
   162     (case TimeLimit.timeLimit time (Seq.pull o full_tac) goal of
   162     (case TimeLimit.timeLimit time (Seq.pull o full_tac) goal of
   163       SOME (thm, _) => true
   163       SOME _ => true
   164     | NONE => false)
   164     | NONE => false)
   165   end
   165   end
   166 
   166 
   167 local
   167 local
   168 
   168