src/HOL/Tools/Sledgehammer/sledgehammer_mash.ML
changeset 50608 5977de2993ac
parent 50588 074e937459b6
child 50610 d9c4fbbb0c11
equal deleted inserted replaced
50607:e928f8647302 50608:5977de2993ac
    56     -> (string * real) list
    56     -> (string * real) list
    57   val isar_dependencies_of : string Symtab.table -> thm -> string list option
    57   val isar_dependencies_of : string Symtab.table -> thm -> string list option
    58   val prover_dependencies_of :
    58   val prover_dependencies_of :
    59     Proof.context -> params -> string -> int -> fact list -> string Symtab.table
    59     Proof.context -> params -> string -> int -> fact list -> string Symtab.table
    60     -> thm -> bool * string list option
    60     -> thm -> bool * string list option
    61   val weight_mash_facts : ('a * thm) list -> (('a * thm) * real) list
    61   val weight_mash_facts : 'a list -> ('a * real) list
    62   val find_mash_suggestions :
    62   val find_mash_suggestions :
    63     int -> (Symtab.key * 'a) list -> ('b * thm) list -> ('b * thm) list
    63     int -> (Symtab.key * 'a) list -> ('b * thm) list -> ('b * thm) list
    64     -> ('b * thm) list -> ('b * thm) list * ('b * thm) list
    64     -> ('b * thm) list -> ('b * thm) list * ('b * thm) list
    65   val mash_suggested_facts :
    65   val mash_suggested_facts :
    66     Proof.context -> params -> string -> int -> term list -> term -> fact list
    66     Proof.context -> params -> string -> int -> term list -> term -> fact list
   725   in find_maxes Symtab.empty ([], Graph.maximals fact_G) end
   725   in find_maxes Symtab.empty ([], Graph.maximals fact_G) end
   726 
   726 
   727 fun is_fact_in_graph fact_G (_, th) =
   727 fun is_fact_in_graph fact_G (_, th) =
   728   can (Graph.get_node fact_G) (nickname_of th)
   728   can (Graph.get_node fact_G) (nickname_of th)
   729 
   729 
   730 (* use MePo weights for now *)
       
   731 val weight_raw_mash_facts = weight_mepo_facts
   730 val weight_raw_mash_facts = weight_mepo_facts
   732 val weight_mash_facts = weight_raw_mash_facts
   731 val weight_mash_facts = weight_raw_mash_facts
   733 
   732 
   734 (* FUDGE *)
   733 (* FUDGE *)
   735 fun weight_of_proximity_fact rank =
   734 fun weight_of_proximity_fact rank =