src/HOL/Tools/Sledgehammer/sledgehammer_atp_systems.ML
changeset 75034 890b70f96fe4
parent 75029 dc6769b86fd6
child 75036 212e9ec706cf
equal deleted inserted replaced
75033:b55d84e41d61 75034:890b70f96fe4
   297            (THF (Monomorphic, {with_ite = false, with_let = false}, THF_Lambda_Free), "mono_native_higher", combsN)
   297            (THF (Monomorphic, {with_ite = false, with_let = false}, THF_Lambda_Free), "mono_native_higher", combsN)
   298      in
   298      in
   299        (* FUDGE *)
   299        (* FUDGE *)
   300        K [((512, meshN), (format, type_enc, lam_trans, false, e_fun_weightN)),
   300        K [((512, meshN), (format, type_enc, lam_trans, false, e_fun_weightN)),
   301         ((1024, meshN), (format, type_enc, lam_trans, false, e_sym_offset_weightN)),
   301         ((1024, meshN), (format, type_enc, lam_trans, false, e_sym_offset_weightN)),
   302         ((91, mepoN), (format, type_enc, lam_trans, false, e_autoN)),
   302         ((128, mepoN), (format, type_enc, lam_trans, false, e_autoN)),
   303         ((1000, meshN), (format, "poly_guards??", lam_trans, false, e_sym_offset_weightN)),
   303         ((724, meshN), (format, "poly_guards??", lam_trans, false, e_sym_offset_weightN)),
   304         ((256, mepoN), (format, type_enc, liftingN, false, e_fun_weightN)),
   304         ((256, mepoN), (format, type_enc, liftingN, false, e_fun_weightN)),
   305         ((64, mashN), (format, type_enc, combsN, false, e_fun_weightN))]
   305         ((64, mashN), (format, type_enc, combsN, false, e_fun_weightN))]
   306      end,
   306      end,
   307    good_max_mono_iters = default_max_mono_iters,
   307    good_max_mono_iters = default_max_mono_iters,
   308    good_max_new_mono_instances = default_max_new_mono_instances}
   308    good_max_new_mono_instances = default_max_new_mono_instances}