src/HOL/Tools/res_atp.ML
changeset 22824 51bb2f6ecc4a
parent 22731 abfdccaed085
child 22865 da52c2bd66ae
equal deleted inserted replaced
22823:fa9ff469247f 22824:51bb2f6ecc4a
    29   val eproverLimit: unit -> int
    29   val eproverLimit: unit -> int
    30   val spassLimit: unit -> int
    30   val spassLimit: unit -> int
    31   val atp_method: (Proof.context -> thm list -> int -> tactic) ->
    31   val atp_method: (Proof.context -> thm list -> int -> tactic) ->
    32     Method.src -> Proof.context -> Proof.method
    32     Method.src -> Proof.context -> Proof.method
    33   val cond_rm_tmp: string -> unit
    33   val cond_rm_tmp: string -> unit
    34   val hol_full_types: unit -> unit
       
    35   val hol_partial_types: unit -> unit
       
    36   val hol_const_types_only: unit -> unit
       
    37   val hol_no_types: unit -> unit
       
    38   val hol_typ_level: unit -> ResHolClause.type_level
       
    39   val include_all: bool ref
    34   val include_all: bool ref
    40   val run_relevance_filter: bool ref
    35   val run_relevance_filter: bool ref
    41   val run_blacklist_filter: bool ref
    36   val run_blacklist_filter: bool ref
    42   val blacklist: string list ref
    37   val blacklist: string list ref
    43   val add_all : unit -> unit
    38   val add_all : unit -> unit
   131 
   126 
   132 
   127 
   133 fun vampireLimit () = !vampire_time;
   128 fun vampireLimit () = !vampire_time;
   134 fun eproverLimit () = !eprover_time;
   129 fun eproverLimit () = !eprover_time;
   135 fun spassLimit () = !spass_time;
   130 fun spassLimit () = !spass_time;
   136 
       
   137 val hol_full_types = ResHolClause.full_types;
       
   138 val hol_partial_types = ResHolClause.partial_types;
       
   139 val hol_const_types_only = ResHolClause.const_types_only;
       
   140 val hol_no_types = ResHolClause.no_types;
       
   141 fun hol_typ_level () = ResHolClause.find_typ_level ();
       
   142 fun is_typed_hol () =
       
   143     let val tp_level = hol_typ_level()
       
   144     in
       
   145         not (tp_level = ResHolClause.T_NONE)
       
   146     end;
       
   147 
   131 
   148 fun atp_input_file () =
   132 fun atp_input_file () =
   149     let val file = !problem_name
   133     let val file = !problem_name
   150     in
   134     in
   151         if !destdir = "" then File.platform_path (File.tmp_path (Path.basic file))
   135         if !destdir = "" then File.platform_path (File.tmp_path (Path.basic file))