src/HOL/Tools/Sledgehammer/sledgehammer_preplay.ML
changeset 55176 d187a9908e84
parent 55170 cdb9435e3cae
child 55193 78eb7fab3284
equal deleted inserted replaced
55175:56c0d70127a9 55176:d187a9908e84
    87   end
    87   end
    88 
    88 
    89 fun tac_of_method meth type_enc lam_trans ctxt facts =
    89 fun tac_of_method meth type_enc lam_trans ctxt facts =
    90   (case meth of
    90   (case meth of
    91     Metis_Method => Metis_Tactic.metis_tac [type_enc] lam_trans ctxt facts
    91     Metis_Method => Metis_Tactic.metis_tac [type_enc] lam_trans ctxt facts
    92   | Metis_New_Skolem_Method =>
       
    93     tac_of_method Metis_Method type_enc lam_trans (Config.put Metis_Tactic.new_skolem true ctxt)
       
    94       facts
       
    95   | Meson_Method => Meson.meson_tac ctxt facts
    92   | Meson_Method => Meson.meson_tac ctxt facts
    96   | _ =>
    93   | _ =>
    97     Method.insert_tac facts THEN'
    94     Method.insert_tac facts THEN'
    98     (case meth of
    95     (case meth of
    99       Simp_Method => Simplifier.asm_full_simp_tac ctxt
    96       Metis_New_Skolem_Method => Metis_Tactic.metis_tac [type_enc] lam_trans ctxt []
       
    97     | Simp_Method => Simplifier.asm_full_simp_tac ctxt
   100     | Simp_Size_Method =>
    98     | Simp_Size_Method =>
   101       Simplifier.asm_full_simp_tac (Simplifier.add_simp @{thm size_ne_size_imp_ne} ctxt)
    99       Simplifier.asm_full_simp_tac (Simplifier.add_simp @{thm size_ne_size_imp_ne} ctxt)
   102     | Auto_Method => K (Clasimp.auto_tac ctxt)
   100     | Auto_Method => K (Clasimp.auto_tac ctxt)
   103     | Fastforce_Method => Clasimp.fast_force_tac ctxt
   101     | Fastforce_Method => Clasimp.fast_force_tac ctxt
   104     | Force_Method => Clasimp.force_tac ctxt
   102     | Force_Method => Clasimp.force_tac ctxt