src/HOL/Tools/Sledgehammer/sledgehammer_isar_preplay.ML
changeset 55219 6fe9fd75f9d7
parent 55213 dcb36a2540bc
child 55221 ee90eebb8b73
equal deleted inserted replaced
55218:ed495a5088c6 55219:6fe9fd75f9d7
    99     | Auto_Method => K (Clasimp.auto_tac ctxt)
    99     | Auto_Method => K (Clasimp.auto_tac ctxt)
   100     | Fastforce_Method => Clasimp.fast_force_tac ctxt
   100     | Fastforce_Method => Clasimp.fast_force_tac ctxt
   101     | Force_Method => Clasimp.force_tac ctxt
   101     | Force_Method => Clasimp.force_tac ctxt
   102     | Arith_Method => Arith_Data.arith_tac ctxt
   102     | Arith_Method => Arith_Data.arith_tac ctxt
   103     | Blast_Method => blast_tac ctxt
   103     | Blast_Method => blast_tac ctxt
       
   104     | Algebra_Method => Groebner.algebra_tac [] [] ctxt
   104     | _ => raise Fail "Sledgehammer_Isar_Preplay: tac_of_method"))
   105     | _ => raise Fail "Sledgehammer_Isar_Preplay: tac_of_method"))
   105 
   106 
   106 (* main function for preplaying Isar steps; may throw exceptions *)
   107 (* main function for preplaying Isar steps; may throw exceptions *)
   107 fun preplay_raw _ _ _ _ _ (Let _) = Played Time.zeroTime
   108 fun preplay_raw _ _ _ _ _ (Let _) = Played Time.zeroTime
   108   | preplay_raw debug type_enc lam_trans ctxt timeout
   109   | preplay_raw debug type_enc lam_trans ctxt timeout