src/HOL/Tools/Sledgehammer/sledgehammer_atp_systems.ML
changeset 74109 ed1f576df9c4
parent 74047 a2b470e315ee
child 74117 30ab39ab4117
equal deleted inserted replaced
74105:d3d6e01a6b00 74109:ed1f576df9c4
   680                 else combsN, uncurried_aliases), ""))],
   680                 else combsN, uncurried_aliases), ""))],
   681    best_max_mono_iters = default_max_mono_iters,
   681    best_max_mono_iters = default_max_mono_iters,
   682    best_max_new_mono_instances = default_max_new_mono_instances}
   682    best_max_new_mono_instances = default_max_new_mono_instances}
   683 
   683 
   684 val dummy_tfx_format = TFF (With_FOOL, Polymorphic)
   684 val dummy_tfx_format = TFF (With_FOOL, Polymorphic)
   685 
       
   686 val dummy_tfx_config = dummy_config Hypothesis dummy_tfx_format "mono_native_fool" false
   685 val dummy_tfx_config = dummy_config Hypothesis dummy_tfx_format "mono_native_fool" false
   687 val dummy_tfx = (dummy_tfxN, fn () => dummy_tfx_config)
   686 val dummy_tfx = (dummy_tfxN, fn () => dummy_tfx_config)
       
   687 
       
   688 val dummy_thf_format = THF (With_FOOL, Polymorphic, THF_With_Choice)
       
   689 val dummy_thf_config = dummy_config Hypothesis dummy_thf_format "mono_native_higher_fool" false
       
   690 val dummy_thf = (dummy_thfN, fn () => dummy_thf_config)
   688 
   691 
   689 
   692 
   690 (* Setup *)
   693 (* Setup *)
   691 
   694 
   692 fun add_atp (name, config) thy =
   695 fun add_atp (name, config) thy =
   720   end
   723   end
   721 
   724 
   722 val atps =
   725 val atps =
   723   [agsyhol, alt_ergo, e, iprover, leo2, leo3, satallax, spass, vampire, z3_tptp, zipperposition,
   726   [agsyhol, alt_ergo, e, iprover, leo2, leo3, satallax, spass, vampire, z3_tptp, zipperposition,
   724    remote_agsyhol, remote_alt_ergo, remote_e, remote_iprover, remote_leo2, remote_leo3,
   727    remote_agsyhol, remote_alt_ergo, remote_e, remote_iprover, remote_leo2, remote_leo3,
   725    remote_waldmeister, remote_zipperposition, dummy_tfx]
   728    remote_waldmeister, remote_zipperposition, dummy_tfx, dummy_thf]
   726 
   729 
   727 val _ = Theory.setup (fold add_atp atps)
   730 val _ = Theory.setup (fold add_atp atps)
   728 
   731 
   729 end;
   732 end;