| author | traytel | 
| Mon, 11 Aug 2014 10:43:03 +0200 | |
| changeset 57890 | 1e13f63fb452 | 
| parent 57729 | 2df9ed24114f | 
| child 57963 | cb67fac9bd89 | 
| permissions | -rw-r--r-- | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 1 | (* Title: HOL/Tools/Sledgehammer/sledgehammer_fact.ML | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 2 | Author: Jia Meng, Cambridge University Computer Laboratory and NICTA | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 3 | Author: Jasmin Blanchette, TU Muenchen | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 4 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 5 | Sledgehammer fact handling. | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 6 | *) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 7 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 8 | signature SLEDGEHAMMER_FACT = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 9 | sig | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 10 | type status = ATP_Problem_Generate.status | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 11 | type stature = ATP_Problem_Generate.stature | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 12 | |
| 51004 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 13 | type raw_fact = ((unit -> string) * stature) * thm | 
| 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 14 | type fact = (string * stature) * thm | 
| 48296 
e7f01b7e244e
gracefully handle the case of empty theories when going up the accessibility chain
 blanchet parents: 
48292diff
changeset | 15 | |
| 48292 | 16 | type fact_override = | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 17 |     {add : (Facts.ref * Attrib.src list) list,
 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 18 | del : (Facts.ref * Attrib.src list) list, | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 19 | only : bool} | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 20 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 21 | val instantiate_inducts : bool Config.T | 
| 48292 | 22 | val no_fact_override : fact_override | 
| 55212 | 23 | |
| 24 | val fact_of_ref : Proof.context -> unit Symtab.table -> thm list -> status Termtab.table -> | |
| 25 | Facts.ref * Attrib.src list -> ((string * stature) * thm) list | |
| 50047 
45684acf0b94
thread context correctly when printing backquoted facts
 blanchet parents: 
49981diff
changeset | 26 | val backquote_thm : Proof.context -> thm -> string | 
| 50511 
8825c36cb1ce
don't query blacklisted theorems in evaluation driver
 blanchet parents: 
50510diff
changeset | 27 | val is_blacklisted_or_something : Proof.context -> bool -> string -> bool | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 28 | val clasimpset_rule_table_of : Proof.context -> status Termtab.table | 
| 55212 | 29 |   val build_name_tables : (thm -> string) -> ('a * thm) list ->
 | 
| 30 | string Symtab.table * string Symtab.table | |
| 31 | val maybe_instantiate_inducts : Proof.context -> term list -> term -> | |
| 32 | (((unit -> string) * 'a) * thm) list -> (((unit -> string) * 'a) * thm) list | |
| 51004 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 33 | val fact_of_raw_fact : raw_fact -> fact | 
| 55212 | 34 | |
| 35 | val all_facts : Proof.context -> bool -> bool -> unit Symtab.table -> thm list -> thm list -> | |
| 36 | status Termtab.table -> raw_fact list | |
| 37 | val nearly_all_facts : Proof.context -> bool -> fact_override -> unit Symtab.table -> | |
| 38 | status Termtab.table -> thm list -> term list -> term -> raw_fact list | |
| 54142 
5f3c1b445253
no fact subsumption -- this only confuses later code, e.g. 'add:'
 blanchet parents: 
54112diff
changeset | 39 | val drop_duplicate_facts : raw_fact list -> raw_fact list | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 40 | end; | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 41 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 42 | structure Sledgehammer_Fact : SLEDGEHAMMER_FACT = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 43 | struct | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 44 | |
| 50495 
bd9a0028b063
better tautology check -- don't reject "prod_cases3" for example
 blanchet parents: 
50490diff
changeset | 45 | open ATP_Util | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 46 | open ATP_Problem_Generate | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 47 | open Sledgehammer_Util | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 48 | |
| 51004 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 49 | type raw_fact = ((unit -> string) * stature) * thm | 
| 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 50 | type fact = (string * stature) * thm | 
| 48296 
e7f01b7e244e
gracefully handle the case of empty theories when going up the accessibility chain
 blanchet parents: 
48292diff
changeset | 51 | |
| 48292 | 52 | type fact_override = | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 53 |   {add : (Facts.ref * Attrib.src list) list,
 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 54 | del : (Facts.ref * Attrib.src list) list, | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 55 | only : bool} | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 56 | |
| 54080 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 57 | (* gracefully handle huge background theories *) | 
| 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 58 | val max_facts_for_duplicates = 50000 | 
| 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 59 | val max_facts_for_complex_check = 25000 | 
| 54083 
824db6ab3339
crank up limit a bit -- truly huge background theories are still nearly 3 times larger
 blanchet parents: 
54081diff
changeset | 60 | val max_simps_for_clasimpset = 10000 | 
| 54080 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 61 | |
| 53511 
3ea6b9461c55
got rid of another slowdown factor in relevance filter
 blanchet parents: 
53510diff
changeset | 62 | (* experimental feature *) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 63 | val instantiate_inducts = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 64 |   Attrib.setup_config_bool @{binding sledgehammer_instantiate_inducts} (K false)
 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 65 | |
| 48292 | 66 | val no_fact_override = {add = [], del = [], only = false}
 | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 67 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 68 | fun needs_quoting reserved s = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 69 | Symtab.defined reserved s orelse | 
| 50239 | 70 | exists (not o Symbol_Pos.is_identifier) (Long_Name.explode s) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 71 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 72 | fun make_name reserved multi j name = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 73 | (name |> needs_quoting reserved name ? quote) ^ | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 74 |   (if multi then "(" ^ string_of_int j ^ ")" else "")
 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 75 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 76 | fun explode_interval _ (Facts.FromTo (i, j)) = i upto j | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 77 | | explode_interval max (Facts.From i) = i upto i + max - 1 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 78 | | explode_interval _ (Facts.Single i) = [i] | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 79 | |
| 57727 
02a53c1bbb6c
generate backquotes without markup, since this confuses preplay; bump up spying version identifier;
 blanchet parents: 
57469diff
changeset | 80 | val backquote = raw_explode #> map (fn "`" => "\\`" | s => s) #> implode #> enclose "`" "`" | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 81 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 82 | (* unfolding these can yield really huge terms *) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 83 | val risky_defs = @{thms Bit0_def Bit1_def}
 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 84 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 85 | fun is_rec_eq lhs = Term.exists_subterm (curry (op =) (head_of lhs)) | 
| 57468 | 86 | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 87 | fun is_rec_def (@{const Trueprop} $ t) = is_rec_def t
 | 
| 56245 | 88 |   | is_rec_def (@{const Pure.imp} $ _ $ t2) = is_rec_def t2
 | 
| 89 |   | is_rec_def (Const (@{const_name Pure.eq}, _) $ t1 $ t2) = is_rec_eq t1 t2
 | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 90 |   | is_rec_def (Const (@{const_name HOL.eq}, _) $ t1 $ t2) = is_rec_eq t1 t2
 | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 91 | | is_rec_def _ = false | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 92 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 93 | fun is_assum assms th = exists (fn ct => prop_of th aconv term_of ct) assms | 
| 48396 | 94 | fun is_chained chained = member Thm.eq_thm_prop chained | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 95 | |
| 48396 | 96 | fun scope_of_thm global assms chained th = | 
| 97 | if is_chained chained th then Chained | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 98 | else if global then Global | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 99 | else if is_assum assms th then Assum | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 100 | else Local | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 101 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 102 | val may_be_induction = | 
| 57729 | 103 |   exists_subterm (fn Var (_, Type (@{type_name fun}, [_, T])) => body_type T = @{typ bool}
 | 
| 104 | | _ => false) | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 105 | |
| 54077 | 106 | (* TODO: get rid of *) | 
| 53501 | 107 | fun normalize_vars t = | 
| 108 | let | |
| 109 | fun normT (Type (s, Ts)) = fold_map normT Ts #>> curry Type s | |
| 110 | | normT (TVar (z as (_, S))) = | |
| 111 | (fn ((knownT, nT), accum) => | |
| 55286 | 112 | (case find_index (equal z) knownT of | 
| 53501 | 113 | ~1 => (TVar ((Name.uu, nT), S), ((z :: knownT, nT + 1), accum)) | 
| 55286 | 114 | | j => (TVar ((Name.uu, nT - j - 1), S), ((knownT, nT), accum)))) | 
| 53501 | 115 | | normT (T as TFree _) = pair T | 
| 57468 | 116 | |
| 53501 | 117 | fun norm (t $ u) = norm t ##>> norm u #>> op $ | 
| 118 | | norm (Const (s, T)) = normT T #>> curry Const s | |
| 57729 | 119 | | norm (Var (z as (_, T))) = normT T | 
| 53501 | 120 | #> (fn (T, (accumT, (known, n))) => | 
| 57729 | 121 | (case find_index (equal z) known of | 
| 122 | ~1 => (Var ((Name.uu, n), T), (accumT, (z :: known, n + 1))) | |
| 123 | | j => (Var ((Name.uu, n - j - 1), T), (accumT, (known, n))))) | |
| 124 | | norm (Abs (_, T, t)) = norm t ##>> normT T #>> (fn (t, T) => Abs (Name.uu, T, t)) | |
| 53501 | 125 | | norm (Bound j) = pair (Bound j) | 
| 126 | | norm (Free (s, T)) = normT T #>> curry Free s | |
| 127 | in fst (norm t (([], 0), ([], 0))) end | |
| 128 | ||
| 48396 | 129 | fun status_of_thm css name th = | 
| 54081 | 130 | if Termtab.is_empty css then | 
| 131 | General | |
| 132 | else | |
| 133 | let val t = prop_of th in | |
| 134 | (* FIXME: use structured name *) | |
| 135 | if String.isSubstring ".induct" name andalso may_be_induction t then | |
| 136 | Induction | |
| 137 | else | |
| 138 | let val t = normalize_vars t in | |
| 55286 | 139 | (case Termtab.lookup css t of | 
| 54081 | 140 | SOME status => status | 
| 141 | | NONE => | |
| 142 | let val concl = Logic.strip_imp_concl t in | |
| 55286 | 143 | (case try (HOLogic.dest_eq o HOLogic.dest_Trueprop) concl of | 
| 54081 | 144 | SOME lrhss => | 
| 145 | let | |
| 146 | val prems = Logic.strip_imp_prems t | |
| 147 | val t' = Logic.list_implies (prems, Logic.mk_equals lrhss) | |
| 148 | in | |
| 149 | Termtab.lookup css t' |> the_default General | |
| 150 | end | |
| 55286 | 151 | | NONE => General) | 
| 152 | end) | |
| 54081 | 153 | end | 
| 154 | end | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 155 | |
| 48396 | 156 | fun stature_of_thm global assms chained css name th = | 
| 157 | (scope_of_thm global assms chained th, status_of_thm css name th) | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 158 | |
| 52031 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 blanchet parents: 
51998diff
changeset | 159 | fun fact_of_ref ctxt reserved chained css (xthm as (xref, args)) = | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 160 | let | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 161 | val ths = Attrib.eval_thms ctxt [xthm] | 
| 57729 | 162 | val bracket = implode (map (enclose "[" "]" o Pretty.str_of o Args.pretty_src ctxt) args) | 
| 57468 | 163 | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 164 | fun nth_name j = | 
| 55286 | 165 | (case xref of | 
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57727diff
changeset | 166 | Facts.Fact s => backquote (simplify_spaces (unyxml s)) ^ bracket | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 167 |       | Facts.Named (("", _), _) => "[" ^ bracket ^ "]"
 | 
| 57729 | 168 | | Facts.Named ((name, _), NONE) => make_name reserved (length ths > 1) (j + 1) name ^ bracket | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 169 | | Facts.Named ((name, _), SOME intervals) => | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 170 | make_name reserved true | 
| 55286 | 171 | (nth (maps (explode_interval (length ths)) intervals) j) name ^ bracket) | 
| 57468 | 172 | |
| 48396 | 173 | fun add_nth th (j, rest) = | 
| 174 | let val name = nth_name j in | |
| 57729 | 175 | (j + 1, ((name, stature_of_thm false [] chained css name th), th) :: rest) | 
| 48396 | 176 | end | 
| 57468 | 177 | in | 
| 178 | (0, []) |> fold add_nth ths |> snd | |
| 179 | end | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 180 | |
| 57729 | 181 | (* Reject theorems with names like "List.filter.filter_list_def" or "Accessible_Part.acc.defs", as | 
| 182 | these are definitions arising from packages. *) | |
| 50736 | 183 | fun is_package_def s = | 
| 184 | let val ss = Long_Name.explode s in | |
| 185 | length ss > 2 andalso not (hd ss = "local") andalso | |
| 186 | exists (fn suf => String.isSuffix suf s) | |
| 57729 | 187 | ["_case_def", "_rec_def", "_size_def", "_size_overloaded_def"] | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 188 | end | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 189 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 190 | (* FIXME: put other record thms here, or declare as "no_atp" *) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 191 | fun multi_base_blacklist ctxt ho_atp = | 
| 57729 | 192 | ["defs", "select_defs", "update_defs", "split", "splits", "split_asm", "ext_cases", "eq.simps", | 
| 193 | "eq.refl", "nchotomy", "case_cong", "weak_case_cong", "nat_of_char_simps", "nibble.simps", | |
| 48440 
159e320ef851
identified "evil" theories for MaSh -- this is rather ad hoc, but so is MaSh anyway
 blanchet parents: 
48438diff
changeset | 194 | "nibble.distinct"] | 
| 57729 | 195 | |> not (ho_atp orelse Config.get ctxt instantiate_inducts) ? append ["induct", "inducts"] | 
| 48440 
159e320ef851
identified "evil" theories for MaSh -- this is rather ad hoc, but so is MaSh anyway
 blanchet parents: 
48438diff
changeset | 196 | |> map (prefix Long_Name.separator) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 197 | |
| 57729 | 198 | (* The maximum apply depth of any "metis" call in "Metis_Examples" (back in 2007) was 11. *) | 
| 53529 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 199 | val max_apply_depth = 18 | 
| 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 200 | |
| 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 201 | fun apply_depth (f $ t) = Int.max (apply_depth f, apply_depth t + 1) | 
| 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 202 | | apply_depth (Abs (_, _, t)) = apply_depth t | 
| 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 203 | | apply_depth _ = 0 | 
| 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 204 | |
| 53533 | 205 | fun is_too_complex t = apply_depth t > max_apply_depth | 
| 53529 
1eb7c65b526c
reverted f99ee3adb81d -- that old logic seems to make a difference still today
 blanchet parents: 
53513diff
changeset | 206 | |
| 48667 
ac58317ef11f
rule out same "technical" theories for MePo as for MaSh
 blanchet parents: 
48530diff
changeset | 207 | (* FIXME: Ad hoc list *) | 
| 
ac58317ef11f
rule out same "technical" theories for MePo as for MaSh
 blanchet parents: 
48530diff
changeset | 208 | val technical_prefixes = | 
| 57729 | 209 | ["ATP", "Code_Evaluation", "Datatype", "Enum", "Lazy_Sequence", "Limited_Sequence", "Meson", | 
| 210 | "Metis", "Nitpick", "Quickcheck_Random", "Quickcheck_Exhaustive", "Quickcheck_Narrowing", | |
| 50736 | 211 | "Random_Sequence", "Sledgehammer", "SMT"] | 
| 48667 
ac58317ef11f
rule out same "technical" theories for MePo as for MaSh
 blanchet parents: 
48530diff
changeset | 212 | |> map (suffix Long_Name.separator) | 
| 48440 
159e320ef851
identified "evil" theories for MaSh -- this is rather ad hoc, but so is MaSh anyway
 blanchet parents: 
48438diff
changeset | 213 | |
| 57729 | 214 | fun is_technical_const s = exists (fn pref => String.isPrefix pref s) technical_prefixes | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 215 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 216 | (* FIXME: make more reliable *) | 
| 53507 | 217 | val sep_class_sep = Long_Name.separator ^ "class" ^ Long_Name.separator | 
| 57468 | 218 | |
| 57729 | 219 | fun is_low_level_class_const s = | 
| 53507 | 220 |   s = @{const_name equal_class.equal} orelse String.isSubstring sep_class_sep s
 | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 221 | |
| 53509 | 222 | val sep_that = Long_Name.separator ^ Obtain.thatN | 
| 54081 | 223 | val skolem_thesis = Name.skolem Auto_Bind.thesisN | 
| 224 | ||
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 225 | fun is_that_fact th = | 
| 54081 | 226 | exists_subterm (fn Free (s, _) => s = skolem_thesis | _ => false) (prop_of th) | 
| 227 | andalso String.isSuffix sep_that (Thm.get_name_hint th) | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 228 | |
| 53513 | 229 | datatype interest = Deal_Breaker | Interesting | Boring | 
| 230 | ||
| 231 | fun combine_interests Deal_Breaker _ = Deal_Breaker | |
| 232 | | combine_interests _ Deal_Breaker = Deal_Breaker | |
| 233 | | combine_interests Interesting _ = Interesting | |
| 234 | | combine_interests _ Interesting = Interesting | |
| 235 | | combine_interests Boring Boring = Boring | |
| 236 | ||
| 54914 
25212efcd0de
removed pointless warning (cf. http://stackoverflow.com/questions/20233463/isabelle-metis-proof-state-contains-the-universal-sort/20785045#20785045)
 blanchet parents: 
54503diff
changeset | 237 | val type_has_top_sort = | 
| 
25212efcd0de
removed pointless warning (cf. http://stackoverflow.com/questions/20233463/isabelle-metis-proof-state-contains-the-universal-sort/20785045#20785045)
 blanchet parents: 
54503diff
changeset | 238 | exists_subtype (fn TFree (_, []) => true | TVar (_, []) => true | _ => false) | 
| 
25212efcd0de
removed pointless warning (cf. http://stackoverflow.com/questions/20233463/isabelle-metis-proof-state-contains-the-universal-sort/20785045#20785045)
 blanchet parents: 
54503diff
changeset | 239 | |
| 50523 
0799339fea0f
get rid of some junk facts in the MaSh evaluation driver
 blanchet parents: 
50512diff
changeset | 240 | fun is_likely_tautology_too_meta_or_too_technical th = | 
| 48406 | 241 | let | 
| 50053 
fea589c8583e
fixed detection of tautologies -- things like "a = b" in a structured proof, where a and b are Frees, shouldn't be discarted as tautologies
 blanchet parents: 
50049diff
changeset | 242 | fun is_interesting_subterm (Const (s, _)) = | 
| 
fea589c8583e
fixed detection of tautologies -- things like "a = b" in a structured proof, where a and b are Frees, shouldn't be discarted as tautologies
 blanchet parents: 
50049diff
changeset | 243 | not (member (op =) atp_widely_irrelevant_consts s) | 
| 
fea589c8583e
fixed detection of tautologies -- things like "a = b" in a structured proof, where a and b are Frees, shouldn't be discarted as tautologies
 blanchet parents: 
50049diff
changeset | 244 | | is_interesting_subterm (Free _) = true | 
| 
fea589c8583e
fixed detection of tautologies -- things like "a = b" in a structured proof, where a and b are Frees, shouldn't be discarted as tautologies
 blanchet parents: 
50049diff
changeset | 245 | | is_interesting_subterm _ = false | 
| 57468 | 246 | |
| 53513 | 247 | fun interest_of_bool t = | 
| 57729 | 248 | if exists_Const ((is_technical_const o fst) orf (is_low_level_class_const o fst) orf | 
| 249 | type_has_top_sort o snd) t then | |
| 53513 | 250 | Deal_Breaker | 
| 251 |       else if exists_type (exists_subtype (curry (op =) @{typ prop})) t orelse
 | |
| 57729 | 252 | not (exists_subterm is_interesting_subterm t) then | 
| 53513 | 253 | Boring | 
| 254 | else | |
| 255 | Interesting | |
| 57468 | 256 | |
| 53513 | 257 |     fun interest_of_prop _ (@{const Trueprop} $ t) = interest_of_bool t
 | 
| 56245 | 258 |       | interest_of_prop Ts (@{const Pure.imp} $ t $ u) =
 | 
| 53513 | 259 | combine_interests (interest_of_prop Ts t) (interest_of_prop Ts u) | 
| 56245 | 260 |       | interest_of_prop Ts (Const (@{const_name Pure.all}, _) $ Abs (_, T, t)) =
 | 
| 54040 | 261 | if type_has_top_sort T then Deal_Breaker else interest_of_prop (T :: Ts) t | 
| 56245 | 262 |       | interest_of_prop Ts ((t as Const (@{const_name Pure.all}, _)) $ u) =
 | 
| 53513 | 263 | interest_of_prop Ts (t $ eta_expand Ts u 1) | 
| 56245 | 264 |       | interest_of_prop _ (Const (@{const_name Pure.eq}, _) $ t $ u) =
 | 
| 53513 | 265 | combine_interests (interest_of_bool t) (interest_of_bool u) | 
| 266 | | interest_of_prop _ _ = Deal_Breaker | |
| 57468 | 267 | |
| 50523 
0799339fea0f
get rid of some junk facts in the MaSh evaluation driver
 blanchet parents: 
50512diff
changeset | 268 | val t = prop_of th | 
| 48406 | 269 | in | 
| 57729 | 270 |     (interest_of_prop [] t <> Interesting andalso not (Thm.eq_thm_prop (@{thm ext}, th))) orelse
 | 
| 53507 | 271 | is_that_fact th | 
| 48438 
3e45c98fe127
distinguish between recursive and nonrecursive definitions + clean up typedef dependencies in MaSh
 blanchet parents: 
48437diff
changeset | 272 | end | 
| 
3e45c98fe127
distinguish between recursive and nonrecursive definitions + clean up typedef dependencies in MaSh
 blanchet parents: 
48437diff
changeset | 273 | |
| 53512 | 274 | fun is_blacklisted_or_something ctxt ho_atp = | 
| 57468 | 275 | let val blist = multi_base_blacklist ctxt ho_atp in | 
| 276 | fn name => is_package_def name orelse exists (fn s => String.isSuffix s name) blist | |
| 277 | end | |
| 50510 | 278 | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 279 | (* This is a terrible hack. Free variables are sometimes coded as "M__" when | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 280 | they are displayed as "M" and we want to avoid clashes with these. But | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 281 | sometimes it's even worse: "Ma__" encodes "M". So we simply reserve all | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 282 | prefixes of all free variables. In the worse case scenario, where the fact | 
| 49981 | 283 | won't be resolved correctly, the user can fix it manually, e.g., by giving a | 
| 284 | name to the offending fact. *) | |
| 57729 | 285 | fun all_prefixes_of s = map (fn i => String.extract (s, 0, SOME i)) (1 upto size s - 1) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 286 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 287 | fun close_form t = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 288 | (t, [] |> Term.add_free_names t |> maps all_prefixes_of) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 289 | |> fold (fn ((s, i), T) => fn (t', taken) => | 
| 57729 | 290 | let val s' = singleton (Name.variant_list taken) s in | 
| 291 | ((if fastype_of t' = HOLogic.boolT then HOLogic.all_const | |
| 292 | else Logic.all_const) T | |
| 293 | $ Abs (s', T, abstract_over (Var ((s, i), T), t')), | |
| 294 | s' :: taken) | |
| 295 | end) | |
| 296 | (Term.add_vars t [] |> sort_wrt (fst o fst)) | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 297 | |> fst | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 298 | |
| 51998 
f732a674db1b
renamed Sledgehammer functions with 'for' in their names to 'of'
 blanchet parents: 
51160diff
changeset | 299 | fun backquote_term ctxt = close_form #> hackish_string_of_term ctxt #> backquote | 
| 
f732a674db1b
renamed Sledgehammer functions with 'for' in their names to 'of'
 blanchet parents: 
51160diff
changeset | 300 | fun backquote_thm ctxt = backquote_term ctxt o prop_of | 
| 48394 
82fc8c956cdc
fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully
 blanchet parents: 
48332diff
changeset | 301 | |
| 54084 | 302 | (* TODO: rewrite to use nets and/or to reuse existing data structures *) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 303 | fun clasimpset_rule_table_of ctxt = | 
| 53502 | 304 | let val simps = ctxt |> simpset_of |> dest_ss |> #simps in | 
| 305 | if length simps >= max_simps_for_clasimpset then | |
| 306 | Termtab.empty | |
| 307 | else | |
| 308 | let | |
| 57729 | 309 | fun add stature th = Termtab.update (normalize_vars (prop_of th), stature) | 
| 57468 | 310 | |
| 57729 | 311 |         val {safeIs, (* safeEs, *) hazIs, (* hazEs, *) ...} = ctxt |> claset_of |> Classical.rep_cs
 | 
| 53502 | 312 | val intros = Item_Net.content safeIs @ Item_Net.content hazIs | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 313 | (* Add once it is used: | 
| 57729 | 314 | val elims = Item_Net.content safeEs @ Item_Net.content hazEs | 
| 53502 | 315 | |> map Classical.classical_rule | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 316 | *) | 
| 57729 | 317 | val specs = Spec_Rules.get ctxt | 
| 318 | val (rec_defs, nonrec_defs) = specs | |
| 319 | |> filter (curry (op =) Spec_Rules.Equational o fst) | |
| 320 | |> maps (snd o snd) | |
| 321 | |> filter_out (member Thm.eq_thm_prop risky_defs) | |
| 322 | |> List.partition (is_rec_def o prop_of) | |
| 323 | val spec_intros = specs | |
| 324 | |> filter (member (op =) [Spec_Rules.Inductive, Spec_Rules.Co_Inductive] o fst) | |
| 325 | |> maps (snd o snd) | |
| 53502 | 326 | in | 
| 57468 | 327 | Termtab.empty | 
| 328 | |> fold (add Simp o snd) simps | |
| 329 | |> fold (add Rec_Def) rec_defs | |
| 330 | |> fold (add Non_Rec_Def) nonrec_defs | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 331 | (* Add once it is used: | 
| 57468 | 332 | |> fold (add Elim) elims | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 333 | *) | 
| 57468 | 334 | |> fold (add Intro) intros | 
| 335 | |> fold (add Inductive) spec_intros | |
| 53502 | 336 | end | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 337 | end | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 338 | |
| 54092 | 339 | fun normalize_eq (@{const Trueprop} $ (t as (t0 as Const (@{const_name HOL.eq}, _)) $ t1 $ t2)) =
 | 
| 340 | if Term_Ord.fast_term_ord (t1, t2) <> GREATER then t else t0 $ t2 $ t1 | |
| 341 |   | normalize_eq (@{const Trueprop} $ (t as @{const Not}
 | |
| 57729 | 342 |       $ ((t0 as Const (@{const_name HOL.eq}, _)) $ t1 $ t2))) =
 | 
| 54092 | 343 | if Term_Ord.fast_term_ord (t1, t2) <> GREATER then t else HOLogic.mk_not (t0 $ t2 $ t1) | 
| 56245 | 344 |   | normalize_eq (Const (@{const_name Pure.eq}, Type (_, [T, _])) $ t1 $ t2) =
 | 
| 54092 | 345 | (if Term_Ord.fast_term_ord (t1, t2) <> GREATER then (t1, t2) else (t2, t1)) | 
| 346 | |> (fn (t1, t2) => HOLogic.eq_const T $ t1 $ t2) | |
| 50481 
5d147d492792
push normalization further -- avoid theorems that are duplicates of each other except for equality symmetry (esp. for "list.distinct(1)" vs. "(2)" etc.)
 blanchet parents: 
50442diff
changeset | 347 | | normalize_eq t = t | 
| 
5d147d492792
push normalization further -- avoid theorems that are duplicates of each other except for equality symmetry (esp. for "list.distinct(1)" vs. "(2)" etc.)
 blanchet parents: 
50442diff
changeset | 348 | |
| 50485 
3c6ac2da2f45
merge aliased theorems in MaSh dependencies, modulo symmetry of equality
 blanchet parents: 
50481diff
changeset | 349 | fun if_thm_before th th' = | 
| 
3c6ac2da2f45
merge aliased theorems in MaSh dependencies, modulo symmetry of equality
 blanchet parents: 
50481diff
changeset | 350 | if Theory.subthy (pairself Thm.theory_of_thm (th, th')) then th else th' | 
| 
3c6ac2da2f45
merge aliased theorems in MaSh dependencies, modulo symmetry of equality
 blanchet parents: 
50481diff
changeset | 351 | |
| 57468 | 352 | (* Hack: Conflate the facts about a class as seen from the outside with the corresponding low-level | 
| 353 | facts, so that MaSh can learn from the low-level proofs. *) | |
| 50734 | 354 | fun un_class_ify s = | 
| 55286 | 355 | (case first_field "_class" s of | 
| 50734 | 356 | SOME (pref, suf) => [s, pref ^ suf] | 
| 55286 | 357 | | NONE => [s]) | 
| 50734 | 358 | |
| 50735 
6b232d76cbc9
refined class handling, to prevent cycles in fact graph
 blanchet parents: 
50734diff
changeset | 359 | fun build_name_tables name_of facts = | 
| 50733 | 360 | let | 
| 54092 | 361 | fun cons_thm (_, th) = Termtab.cons_list (normalize_vars (normalize_eq (prop_of th)), th) | 
| 50735 
6b232d76cbc9
refined class handling, to prevent cycles in fact graph
 blanchet parents: 
50734diff
changeset | 362 | fun add_plain canon alias = | 
| 54092 | 363 | Symtab.update (Thm.get_name_hint alias, name_of (if_thm_before canon alias)) | 
| 50735 
6b232d76cbc9
refined class handling, to prevent cycles in fact graph
 blanchet parents: 
50734diff
changeset | 364 | fun add_plains (_, aliases as canon :: _) = fold (add_plain canon) aliases | 
| 54092 | 365 | fun add_inclass (name, target) = fold (fn s => Symtab.update (s, target)) (un_class_ify name) | 
| 50815 | 366 | val prop_tab = fold cons_thm facts Termtab.empty | 
| 50735 
6b232d76cbc9
refined class handling, to prevent cycles in fact graph
 blanchet parents: 
50734diff
changeset | 367 | val plain_name_tab = Termtab.fold add_plains prop_tab Symtab.empty | 
| 
6b232d76cbc9
refined class handling, to prevent cycles in fact graph
 blanchet parents: 
50734diff
changeset | 368 | val inclass_name_tab = Symtab.fold add_inclass plain_name_tab Symtab.empty | 
| 57108 
dc0b4f50e288
more generous max number of suggestions, for more safety
 blanchet parents: 
56245diff
changeset | 369 | in | 
| 
dc0b4f50e288
more generous max number of suggestions, for more safety
 blanchet parents: 
56245diff
changeset | 370 | (plain_name_tab, inclass_name_tab) | 
| 
dc0b4f50e288
more generous max number of suggestions, for more safety
 blanchet parents: 
56245diff
changeset | 371 | end | 
| 50485 
3c6ac2da2f45
merge aliased theorems in MaSh dependencies, modulo symmetry of equality
 blanchet parents: 
50481diff
changeset | 372 | |
| 54080 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 373 | fun fact_distinct eq facts = | 
| 54076 | 374 | fold (fn fact as (_, th) => | 
| 54080 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 375 | Net.insert_term_safe (eq o pairself (normalize_eq o prop_of o snd)) | 
| 54077 | 376 | (normalize_eq (prop_of th), fact)) | 
| 377 | facts Net.empty | |
| 54076 | 378 | |> Net.entries | 
| 53504 | 379 | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 380 | fun struct_induct_rule_on th = | 
| 55286 | 381 | (case Logic.strip_horn (prop_of th) of | 
| 57729 | 382 |     (prems, @{const Trueprop} $ ((p as Var ((p_name, 0), _)) $ (a as Var (_, ind_T)))) =>
 | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 383 | if not (is_TVar ind_T) andalso length prems > 1 andalso | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 384 | exists (exists_subterm (curry (op aconv) p)) prems andalso | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 385 | not (exists (exists_subterm (curry (op aconv) a)) prems) then | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 386 | SOME (p_name, ind_T) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 387 | else | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 388 | NONE | 
| 55286 | 389 | | _ => NONE) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 390 | |
| 50586 | 391 | val instantiate_induct_timeout = seconds 0.01 | 
| 392 | ||
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 393 | fun instantiate_induct_rule ctxt concl_prop p_name ((name, stature), th) ind_x = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 394 | let | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 395 | fun varify_noninducts (t as Free (s, T)) = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 396 | if (s, T) = ind_x orelse can dest_funT T then t else Var ((s, 0), T) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 397 | | varify_noninducts t = t | 
| 57468 | 398 | |
| 57729 | 399 | val p_inst = concl_prop | 
| 400 | |> map_aterms varify_noninducts | |
| 401 | |> close_form | |
| 402 | |> lambda (Free ind_x) | |
| 403 | |> hackish_string_of_term ctxt | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 404 | in | 
| 57729 | 405 | ((fn () => name () ^ "[where " ^ p_name ^ " = " ^ quote p_inst ^ "]", stature), | 
| 406 | th |> Rule_Insts.read_instantiate ctxt [((p_name, 0), p_inst)] []) | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 407 | end | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 408 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 409 | fun type_match thy (T1, T2) = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 410 | (Sign.typ_match thy (T2, T1) Vartab.empty; true) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 411 | handle Type.TYPE_MATCH => false | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 412 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 413 | fun instantiate_if_induct_rule ctxt stmt stmt_xs (ax as (_, th)) = | 
| 55286 | 414 | (case struct_induct_rule_on th of | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 415 | SOME (p_name, ind_T) => | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 416 | let val thy = Proof_Context.theory_of ctxt in | 
| 55286 | 417 | stmt_xs | 
| 418 | |> filter (fn (_, T) => type_match thy (T, ind_T)) | |
| 419 | |> map_filter (try (TimeLimit.timeLimit instantiate_induct_timeout | |
| 57729 | 420 | (instantiate_induct_rule ctxt stmt p_name ax))) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 421 | end | 
| 55286 | 422 | | NONE => [ax]) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 423 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 424 | fun external_frees t = | 
| 55948 | 425 | [] |> Term.add_frees t |> filter_out (Name.is_internal o fst) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 426 | |
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 427 | fun maybe_instantiate_inducts ctxt hyp_ts concl_t = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 428 | if Config.get ctxt instantiate_inducts then | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 429 | let | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 430 | val thy = Proof_Context.theory_of ctxt | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 431 | val ind_stmt = | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 432 | (hyp_ts |> filter_out (null o external_frees), concl_t) | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 433 | |> Logic.list_implies |> Object_Logic.atomize_term thy | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 434 | val ind_stmt_xs = external_frees ind_stmt | 
| 57729 | 435 | in | 
| 436 | maps (instantiate_if_induct_rule ctxt ind_stmt ind_stmt_xs) | |
| 437 | end | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 438 | else | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 439 | I | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 440 | |
| 51004 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 441 | fun fact_of_raw_fact ((name, stature), th) = ((name (), stature), th) | 
| 
5f2788c38127
distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds
 blanchet parents: 
50815diff
changeset | 442 | |
| 53532 
4ad9599a0847
disable some checks for huge background theories
 blanchet parents: 
53531diff
changeset | 443 | fun fact_count facts = Facts.fold_static (K (Integer.add 1)) facts 0 | 
| 
4ad9599a0847
disable some checks for huge background theories
 blanchet parents: 
53531diff
changeset | 444 | |
| 50523 
0799339fea0f
get rid of some junk facts in the MaSh evaluation driver
 blanchet parents: 
50512diff
changeset | 445 | fun all_facts ctxt generous ho_atp reserved add_ths chained css = | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 446 | let | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 447 | val thy = Proof_Context.theory_of ctxt | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 448 | val global_facts = Global_Theory.facts_of thy | 
| 53532 
4ad9599a0847
disable some checks for huge background theories
 blanchet parents: 
53531diff
changeset | 449 | val is_too_complex = | 
| 57729 | 450 | if generous orelse fact_count global_facts >= max_facts_for_complex_check then K false | 
| 451 | else is_too_complex | |
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 452 | val local_facts = Proof_Context.facts_of ctxt | 
| 56158 
c2c6d560e7b2
more explicit treatment of verbose mode, which includes concealed entries;
 wenzelm parents: 
56141diff
changeset | 453 | val named_locals = local_facts |> Facts.dest_static true [global_facts] | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 454 | val assms = Assumption.all_assms_of ctxt | 
| 57468 | 455 | |
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 456 | fun is_good_unnamed_local th = | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 457 | not (Thm.has_name_hint th) andalso | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 458 | forall (fn (_, ths) => not (member Thm.eq_thm_prop ths th)) named_locals | 
| 57468 | 459 | |
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 460 | val unnamed_locals = | 
| 48396 | 461 | union Thm.eq_thm_prop (Facts.props local_facts) chained | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 462 | |> filter is_good_unnamed_local |> map (pair "" o single) | 
| 57729 | 463 | val full_space = Name_Space.merge (Facts.space_of global_facts, Facts.space_of local_facts) | 
| 53512 | 464 | val is_blacklisted_or_something = is_blacklisted_or_something ctxt ho_atp | 
| 57468 | 465 | |
| 56141 
c06202417c4a
back to a form of hybrid facts, to reduce performance impact of ed92ce2ac88e;
 wenzelm parents: 
56140diff
changeset | 466 | fun add_facts global foldx facts = | 
| 54081 | 467 | foldx (fn (name0, ths) => fn accum => | 
| 50512 
c283bc0a8f1a
tweaked which facts are included for MaSh evaluations
 blanchet parents: 
50511diff
changeset | 468 | if name0 <> "" andalso | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 469 | forall (not o member Thm.eq_thm_prop add_ths) ths andalso | 
| 56141 
c06202417c4a
back to a form of hybrid facts, to reduce performance impact of ed92ce2ac88e;
 wenzelm parents: 
56140diff
changeset | 470 | (Facts.is_concealed facts name0 orelse | 
| 57469 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 471 | Long_Name.is_hidden (Facts.intern facts name0) orelse | 
| 53512 | 472 | (not generous andalso is_blacklisted_or_something name0)) then | 
| 54081 | 473 | accum | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 474 | else | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 475 | let | 
| 50485 
3c6ac2da2f45
merge aliased theorems in MaSh dependencies, modulo symmetry of equality
 blanchet parents: 
50481diff
changeset | 476 | val n = length ths | 
| 
3c6ac2da2f45
merge aliased theorems in MaSh dependencies, modulo symmetry of equality
 blanchet parents: 
50481diff
changeset | 477 | val multi = n > 1 | 
| 57468 | 478 | |
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 479 | fun check_thms a = | 
| 55286 | 480 | (case try (Proof_Context.get_thms ctxt) a of | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 481 | NONE => false | 
| 55286 | 482 | | SOME ths' => eq_list Thm.eq_thm_prop (ths, ths')) | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 483 | in | 
| 57469 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 484 | snd (fold_rev (fn th => fn (j, accum) => | 
| 54081 | 485 | (j - 1, | 
| 486 | if not (member Thm.eq_thm_prop add_ths th) andalso | |
| 487 | (is_likely_tautology_too_meta_or_too_technical th orelse | |
| 488 | is_too_complex (prop_of th)) then | |
| 489 | accum | |
| 490 | else | |
| 491 | let | |
| 57469 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 492 | fun get_name () = | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 493 | if name0 = "" then | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 494 | backquote_thm ctxt th | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 495 | else | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 496 | let val short_name = Facts.extern ctxt facts name0 in | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 497 | if check_thms short_name then | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 498 | short_name | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 499 | else | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 500 | let val long_name = Name_Space.extern ctxt full_space name0 in | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 501 | if check_thms long_name then | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 502 | long_name | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 503 | else | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 504 | name0 | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 505 | end | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 506 | end | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 507 | |> make_name reserved multi j | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 508 | val stature = stature_of_thm global assms chained css name0 th | 
| 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 509 | val new = ((get_name, stature), th) | 
| 54081 | 510 | in | 
| 57469 
29e7e6e89a0e
added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'
 blanchet parents: 
57468diff
changeset | 511 | (if multi then apsnd else apfst) (cons new) accum | 
| 54081 | 512 | end)) ths (n, accum)) | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 513 | end) | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 514 | in | 
| 57729 | 515 | (* The single-theorem names go before the multiple-theorem ones (e.g., "xxx" vs. "xxx(3)"), so | 
| 516 | that single names are preferred when both are available. *) | |
| 517 | `I [] | |
| 518 | |> add_facts false fold local_facts (unnamed_locals @ named_locals) | |
| 519 | |> add_facts true Facts.fold_static global_facts global_facts | |
| 520 | |> op @ | |
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 521 | end | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48250diff
changeset | 522 | |
| 57468 | 523 | fun nearly_all_facts ctxt ho_atp {add, del, only} reserved css chained hyp_ts concl_t =
 | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 524 | if only andalso null add then | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 525 | [] | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 526 | else | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 527 | let | 
| 57729 | 528 | val chained = chained |> maps (fn th => insert Thm.eq_thm_prop (zero_var_indexes th) [th]) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 529 | in | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 530 | (if only then | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 531 | maps (map (fn ((name, stature), th) => ((K name, stature), th)) | 
| 57729 | 532 | o fact_of_ref ctxt reserved chained css) add | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 533 | else | 
| 54080 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 534 | let | 
| 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 535 | val (add, del) = pairself (Attrib.eval_thms ctxt) (add, del) | 
| 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 536 | val facts = | 
| 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 537 | all_facts ctxt false ho_atp reserved add chained css | 
| 54143 
18def1c73c79
make sure add: doesn't add duplicates, and works for [no_atp] facts
 blanchet parents: 
54142diff
changeset | 538 | |> filter_out ((member Thm.eq_thm_prop del orf | 
| 
18def1c73c79
make sure add: doesn't add duplicates, and works for [no_atp] facts
 blanchet parents: 
54142diff
changeset | 539 | (No_ATPs.member ctxt andf not o member Thm.eq_thm_prop add)) o snd) | 
| 54080 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 540 | in | 
| 
540835cf11ed
more gracefully handle huge theories in relevance filters
 blanchet parents: 
54078diff
changeset | 541 | facts | 
| 48292 | 542 | end) | 
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 543 | |> maybe_instantiate_inducts ctxt hyp_ts concl_t | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 544 | end | 
| 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 545 | |
| 54142 
5f3c1b445253
no fact subsumption -- this only confuses later code, e.g. 'add:'
 blanchet parents: 
54112diff
changeset | 546 | fun drop_duplicate_facts facts = | 
| 54112 
9c0f464d1854
drop only real duplicates, not subsumed facts -- this confuses MaSh
 blanchet parents: 
54092diff
changeset | 547 | let val num_facts = length facts in | 
| 54142 
5f3c1b445253
no fact subsumption -- this only confuses later code, e.g. 'add:'
 blanchet parents: 
54112diff
changeset | 548 | facts |> num_facts <= max_facts_for_duplicates ? fact_distinct (op aconv) | 
| 54112 
9c0f464d1854
drop only real duplicates, not subsumed facts -- this confuses MaSh
 blanchet parents: 
54092diff
changeset | 549 | end | 
| 
9c0f464d1854
drop only real duplicates, not subsumed facts -- this confuses MaSh
 blanchet parents: 
54092diff
changeset | 550 | |
| 48250 
1065c307fafe
further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)
 blanchet parents: diff
changeset | 551 | end; |