src/HOL/Tools/Sledgehammer/sledgehammer_provers.ML
changeset 46320 0b8b73b49848
parent 46301 e2e52c7d25c9
child 46340 cac402c486b0
equal deleted inserted replaced
46319:c248e4f1be74 46320:0b8b73b49848
     7 *)
     7 *)
     8 
     8 
     9 signature SLEDGEHAMMER_PROVERS =
     9 signature SLEDGEHAMMER_PROVERS =
    10 sig
    10 sig
    11   type failure = ATP_Proof.failure
    11   type failure = ATP_Proof.failure
    12   type locality = ATP_Translate.locality
    12   type locality = ATP_Problem_Generate.locality
    13   type type_enc = ATP_Translate.type_enc
    13   type type_enc = ATP_Problem_Generate.type_enc
    14   type reconstructor = ATP_Reconstruct.reconstructor
    14   type reconstructor = ATP_Proof_Reconstruct.reconstructor
    15   type play = ATP_Reconstruct.play
    15   type play = ATP_Proof_Reconstruct.play
    16   type minimize_command = ATP_Reconstruct.minimize_command
    16   type minimize_command = ATP_Proof_Reconstruct.minimize_command
    17   type relevance_fudge = Sledgehammer_Filter.relevance_fudge
    17   type relevance_fudge = Sledgehammer_Filter.relevance_fudge
    18 
    18 
    19   datatype mode = Auto_Try | Try | Normal | Auto_Minimize | Minimize
    19   datatype mode = Auto_Try | Try | Normal | Auto_Minimize | Minimize
    20 
    20 
    21   type params =
    21   type params =
   117 
   117 
   118 open ATP_Util
   118 open ATP_Util
   119 open ATP_Problem
   119 open ATP_Problem
   120 open ATP_Proof
   120 open ATP_Proof
   121 open ATP_Systems
   121 open ATP_Systems
   122 open ATP_Translate
   122 open ATP_Problem_Generate
   123 open ATP_Reconstruct
   123 open ATP_Proof_Reconstruct
   124 open Metis_Tactic
   124 open Metis_Tactic
   125 open Sledgehammer_Util
   125 open Sledgehammer_Util
   126 open Sledgehammer_Filter
   126 open Sledgehammer_Filter
   127 
   127 
   128 (** The Sledgehammer **)
   128 (** The Sledgehammer **)