src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
changeset 62519 a564458f94db
parent 62095 7edf47be2baf
child 63337 ae9330fdbc16
equal deleted inserted replaced
62518:b8efcc9edd7b 62519:a564458f94db
   416   (case struct_induct_rule_on th of
   416   (case struct_induct_rule_on th of
   417     SOME (p_name, ind_T) =>
   417     SOME (p_name, ind_T) =>
   418     let val thy = Proof_Context.theory_of ctxt in
   418     let val thy = Proof_Context.theory_of ctxt in
   419       stmt_xs
   419       stmt_xs
   420       |> filter (fn (_, T) => type_match thy (T, ind_T))
   420       |> filter (fn (_, T) => type_match thy (T, ind_T))
   421       |> map_filter (try (TimeLimit.timeLimit instantiate_induct_timeout
   421       |> map_filter (try (Timeout.apply instantiate_induct_timeout
   422         (instantiate_induct_rule ctxt stmt p_name ax)))
   422         (instantiate_induct_rule ctxt stmt p_name ax)))
   423     end
   423     end
   424   | NONE => [ax])
   424   | NONE => [ax])
   425 
   425 
   426 fun external_frees t =
   426 fun external_frees t =