Theory Auto2_HOL_Extra_Setup

(*
  File: Auto2_HOL_Extra_Setup.thy
  Author: Kevin Kappelmann

  Extra setup files for auto2 in HOL.
*)

theory Auto2_HOL_Extra_Setup
  imports
    HOL.HOL
    Auto2_Setup
begin

ML_file ‹acdata.ML›
ML_file ‹ac_steps.ML›
ML_file ‹unfolding.ML›
ML_file ‹induct_outer.ML›
ML_file ‹extra_hol.ML›
ML_file ‹auto2_hol_extra_setup.ML›

end