src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
changeset 55294 6f77310a0907
parent 55288 1a4358d14ce2
child 55296 1d3dadda13a1
equal deleted inserted replaced
55293:42cf5802d36a 55294:6f77310a0907
   135           atp_proof, goal) = try isar_params ()
   135           atp_proof, goal) = try isar_params ()
   136 
   136 
   137         val metislike_methods = insert (op =) (Metis_Method alt_metis_args) metislike_methods0
   137         val metislike_methods = insert (op =) (Metis_Method alt_metis_args) metislike_methods0
   138 
   138 
   139         fun massage_meths (meths as meth :: _) =
   139         fun massage_meths (meths as meth :: _) =
   140           if not try0_isar then [meth]
   140           if not try0_isar then [meth] else if smt then SMT_Method :: meths else meths
   141           else if smt then SMT_Method :: meths
       
   142           else meths
       
   143 
   141 
   144         val (params, _, concl_t) = strip_subgoal goal subgoal ctxt
   142         val (params, _, concl_t) = strip_subgoal goal subgoal ctxt
   145         val fixes = map (fn (s, T) => (Binding.name s, SOME T, NoSyn)) params
   143         val fixes = map (fn (s, T) => (Binding.name s, SOME T, NoSyn)) params
   146         val ctxt = ctxt |> Variable.set_body false |> Proof_Context.add_fixes fixes |> snd
   144         val ctxt = ctxt |> Variable.set_body false |> Proof_Context.add_fixes fixes |> snd
   147 
   145