src/HOL/Tools/Sledgehammer/sledgehammer_prover.ML
changeset 79942 7793e3161d2b
parent 78695 41273636a82a
equal deleted inserted replaced
79941:6a3212bedfad 79942:7793e3161d2b
   216 fun bunches_of_proof_methods ctxt smt_proofs needs_full_types desperate_lam_trans =
   216 fun bunches_of_proof_methods ctxt smt_proofs needs_full_types desperate_lam_trans =
   217   let
   217   let
   218     val misc_methodss =
   218     val misc_methodss =
   219       [[Simp_Method, Auto_Method, Blast_Method, Linarith_Method, Meson_Method,
   219       [[Simp_Method, Auto_Method, Blast_Method, Linarith_Method, Meson_Method,
   220         Metis_Method (NONE, NONE), Fastforce_Method, Force_Method, Presburger_Method,
   220         Metis_Method (NONE, NONE), Fastforce_Method, Force_Method, Presburger_Method,
   221         Argo_Method]]
   221         Argo_Method, Order_Method]]
   222 
   222 
   223     val metis_methodss =
   223     val metis_methodss =
   224       [Metis_Method (SOME full_typesN, NONE) ::
   224       [Metis_Method (SOME full_typesN, NONE) ::
   225        Metis_Method (SOME really_full_type_enc, SOME desperate_lam_trans) ::
   225        Metis_Method (SOME really_full_type_enc, SOME desperate_lam_trans) ::
   226        (if needs_full_types then
   226        (if needs_full_types then