| author | wenzelm | 
| Thu, 09 Jun 2016 15:41:49 +0200 | |
| changeset 63270 | 7dd3ee7ee422 | 
| parent 61770 | a20048c78891 | 
| child 66020 | a31760eee09d | 
| permissions | -rw-r--r-- | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 1 | (* Title: HOL/Tools/ATP/atp_util.ML | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 2 | Author: Jasmin Blanchette, TU Muenchen | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 3 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 4 | General-purpose functions used by the ATP module. | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 5 | *) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 6 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 7 | signature ATP_UTIL = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 8 | sig | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 9 | val timestamp : unit -> string | 
| 53514 | 10 | val hashw : word * word -> word | 
| 11 | val hashw_string : string * word -> word | |
| 43827 
62d64709af3b
added option to control which lambda translation to use (for experiments)
 blanchet parents: 
43572diff
changeset | 12 | val hash_string : string -> int | 
| 48323 | 13 | val chunk_list : int -> 'a list -> 'a list list | 
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48247diff
changeset | 14 | val stringN_of_int : int -> int -> string | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 15 | val strip_spaces : bool -> (char -> bool) -> string -> string | 
| 44784 | 16 | val strip_spaces_except_between_idents : string -> string | 
| 48316 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 17 | val elide_string : int -> string -> string | 
| 52077 | 18 | val find_enclosed : string -> string -> string -> string list | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 19 | val nat_subscript : int -> string | 
| 52076 
bfa28e1cba77
freeze types in Sledgehammer goal, not just terms
 blanchet parents: 
52031diff
changeset | 20 | val unquote_tvar : string -> string | 
| 58928 
23d0ffd48006
plain value Keywords.keywords, which might be used outside theory for bootstrap purposes;
 wenzelm parents: 
58919diff
changeset | 21 | val maybe_quote : Keyword.keywords -> string -> string | 
| 52031 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 blanchet parents: 
51209diff
changeset | 22 | val string_of_ext_time : bool * Time.time -> string | 
| 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 blanchet parents: 
51209diff
changeset | 23 | val string_of_time : Time.time -> string | 
| 47150 | 24 | val type_instance : theory -> typ -> typ -> bool | 
| 25 | val type_generalization : theory -> typ -> typ -> bool | |
| 26 | val type_intersect : theory -> typ -> typ -> bool | |
| 27 | val type_equiv : theory -> typ * typ -> bool | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 28 | val varify_type : Proof.context -> typ -> typ | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 29 | val instantiate_type : theory -> typ -> typ -> typ -> typ | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 30 | val varify_and_instantiate_type : Proof.context -> typ -> typ -> typ -> typ | 
| 44393 | 31 | val is_type_surely_finite : Proof.context -> typ -> bool | 
| 44399 | 32 | val is_type_surely_infinite : Proof.context -> bool -> typ list -> typ -> bool | 
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 33 | val s_not : term -> term | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 34 | val s_conj : term * term -> term | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 35 | val s_disj : term * term -> term | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 36 | val s_imp : term * term -> term | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 37 | val s_iff : term * term -> term | 
| 49983 
33e18e9916a8
use metaquantification when possible in Isar proofs
 blanchet parents: 
49982diff
changeset | 38 | val close_form : term -> term | 
| 49982 | 39 | val hol_close_form_prefix : string | 
| 40 | val hol_close_form : term -> term | |
| 41 | val hol_open_form : (string -> string) -> term -> term | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 42 | val eta_expand : typ list -> term -> int -> term | 
| 59632 | 43 | val cong_extensionalize_term : Proof.context -> term -> term | 
| 47953 
a2c3706c4cb1
added "ext_cong_neq" lemma (not used yet); tuning
 blanchet parents: 
47718diff
changeset | 44 | val abs_extensionalize_term : Proof.context -> term -> term | 
| 47991 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 45 | val unextensionalize_def : term -> term | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 46 | val transform_elim_prop : term -> term | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 47 | val specialize_type : theory -> (string * typ) -> term -> term | 
| 56104 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 48 | val strip_subgoal : thm -> int -> Proof.context -> (string * typ) list * term list * term | 
| 57541 | 49 | val extract_lambda_def : (term -> string * typ) -> term -> string * term | 
| 56104 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 50 | val short_thm_name : Proof.context -> thm -> string | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 51 | end; | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 52 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 53 | structure ATP_Util : ATP_UTIL = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 54 | struct | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 55 | |
| 53800 | 56 | fun timestamp_format time = | 
| 57 | Date.fmt "%Y-%m-%d %H:%M:%S." (Date.fromTimeLocal time) ^ | |
| 58 | (StringCvt.padLeft #"0" 3 (string_of_int (Time.toMilliseconds time - 1000 * Time.toSeconds time))) | |
| 59 | ||
| 60 | val timestamp = timestamp_format o Time.now | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 61 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 62 | (* This hash function is recommended in "Compilers: Principles, Techniques, and | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 63 | Tools" by Aho, Sethi, and Ullman. The "hashpjw" function, which they | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 64 | particularly recommend, triggers a bug in versions of Poly/ML up to 4.2.0. *) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 65 | fun hashw (u, w) = Word.+ (u, Word.* (0w65599, w)) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 66 | fun hashw_char (c, w) = hashw (Word.fromInt (Char.ord c), w) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 67 | fun hashw_string (s : string, w) = CharVector.foldl hashw_char w s | 
| 43827 
62d64709af3b
added option to control which lambda translation to use (for experiments)
 blanchet parents: 
43572diff
changeset | 68 | fun hash_string s = Word.toInt (hashw_string (s, 0w0)) | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 69 | |
| 48323 | 70 | fun chunk_list _ [] = [] | 
| 71 | | chunk_list k xs = | |
| 72 | let val (xs1, xs2) = chop k xs in xs1 :: chunk_list k xs2 end | |
| 73 | ||
| 48251 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48247diff
changeset | 74 | fun stringN_of_int 0 _ = "" | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48247diff
changeset | 75 | | stringN_of_int k n = | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48247diff
changeset | 76 | stringN_of_int (k - 1) (n div 10) ^ string_of_int (n mod 10) | 
| 
6cdcfbddc077
moved most of MaSh exporter code to Sledgehammer
 blanchet parents: 
48247diff
changeset | 77 | |
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 78 | fun is_spaceish c = Char.isSpace c orelse c = #"\127" (* DEL -- no idea where these come from *) | 
| 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 79 | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 80 | fun strip_spaces skip_comments is_evil = | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 81 | let | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 82 | fun strip_c_style_comment [] accum = accum | 
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 83 | | strip_c_style_comment (#"*" :: #"/" :: cs) accum = strip_spaces_in_list true cs accum | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 84 | | strip_c_style_comment (_ :: cs) accum = strip_c_style_comment cs accum | 
| 48766 
553ad5f99968
fixed "double rev" bug that arose in situations where a % comment arose on the last line of a file without \n at the end
 blanchet parents: 
48323diff
changeset | 85 | and strip_spaces_in_list _ [] accum = accum | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 86 | | strip_spaces_in_list true (#"%" :: cs) accum = | 
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 87 | strip_spaces_in_list true (cs |> take_prefix (not_equal #"\n") |> snd) accum | 
| 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 88 | | strip_spaces_in_list true (#"/" :: #"*" :: cs) accum = strip_c_style_comment cs accum | 
| 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 89 | | strip_spaces_in_list _ [c1] accum = accum |> not (is_spaceish c1) ? cons c1 | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 90 | | strip_spaces_in_list skip_comments (cs as [_, _]) accum = | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 91 | accum |> fold (strip_spaces_in_list skip_comments o single) cs | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 92 | | strip_spaces_in_list skip_comments (c1 :: c2 :: c3 :: cs) accum = | 
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 93 | if is_spaceish c1 then | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 94 | strip_spaces_in_list skip_comments (c2 :: c3 :: cs) accum | 
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 95 | else if is_spaceish c2 then | 
| 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 96 | if is_spaceish c3 then | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 97 | strip_spaces_in_list skip_comments (c1 :: c3 :: cs) accum | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 98 | else | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 99 | strip_spaces_in_list skip_comments (c3 :: cs) | 
| 57728 
c21e7bdb40ad
remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer
 blanchet parents: 
57547diff
changeset | 100 | (c1 :: accum |> forall is_evil [c1, c3] ? cons #" ") | 
| 44935 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 101 | else | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 102 | strip_spaces_in_list skip_comments (c2 :: c3 :: cs) (cons c1 accum) | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 103 | in | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 104 | String.explode | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 105 | #> rpair [] #-> strip_spaces_in_list skip_comments | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 106 | #> rev #> String.implode | 
| 
2e812384afa8
tail recursive proof preprocessing (needed for huge proofs)
 blanchet parents: 
44893diff
changeset | 107 | end | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 108 | |
| 44784 | 109 | fun is_ident_char c = Char.isAlphaNum c orelse c = #"_" | 
| 110 | val strip_spaces_except_between_idents = strip_spaces true is_ident_char | |
| 111 | ||
| 48316 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 112 | fun elide_string threshold s = | 
| 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 113 | if size s > threshold then | 
| 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 114 | String.extract (s, 0, SOME (threshold div 2 - 5)) ^ " ...... " ^ | 
| 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 115 | String.extract (s, size s - (threshold + 1) div 2 + 6, NONE) | 
| 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 116 | else | 
| 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 117 | s | 
| 
252f45c04042
drastic overhaul of MaSh data structures + fixed a few performance issues
 blanchet parents: 
48251diff
changeset | 118 | |
| 52077 | 119 | fun find_enclosed left right s = | 
| 120 | case first_field left s of | |
| 121 | SOME (_, s) => | |
| 122 | (case first_field right s of | |
| 123 | SOME (enclosed, s) => enclosed :: find_enclosed left right s | |
| 124 | | NONE => []) | |
| 125 | | NONE => [] | |
| 126 | ||
| 53015 
a1119cf551e8
standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
 wenzelm parents: 
52196diff
changeset | 127 | val subscript = implode o map (prefix "\<^sub>") o raw_explode (* FIXME Symbol.explode (?) *) | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 128 | fun nat_subscript n = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 129 | n |> string_of_int |> print_mode_active Symbol.xsymbolsN ? subscript | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 130 | |
| 52076 
bfa28e1cba77
freeze types in Sledgehammer goal, not just terms
 blanchet parents: 
52031diff
changeset | 131 | val unquote_tvar = perhaps (try (unprefix "'")) | 
| 
bfa28e1cba77
freeze types in Sledgehammer goal, not just terms
 blanchet parents: 
52031diff
changeset | 132 | val unquery_var = perhaps (try (unprefix "?")) | 
| 
bfa28e1cba77
freeze types in Sledgehammer goal, not just terms
 blanchet parents: 
52031diff
changeset | 133 | |
| 50239 | 134 | val is_long_identifier = forall Symbol_Pos.is_identifier o Long_Name.explode | 
| 58928 
23d0ffd48006
plain value Keywords.keywords, which might be used outside theory for bootstrap purposes;
 wenzelm parents: 
58919diff
changeset | 135 | fun maybe_quote keywords y = | 
| 59433 | 136 | let val s = YXML.content_of y in | 
| 52076 
bfa28e1cba77
freeze types in Sledgehammer goal, not just terms
 blanchet parents: 
52031diff
changeset | 137 | y |> ((not (is_long_identifier (unquote_tvar s)) andalso | 
| 
bfa28e1cba77
freeze types in Sledgehammer goal, not just terms
 blanchet parents: 
52031diff
changeset | 138 | not (is_long_identifier (unquery_var s))) orelse | 
| 58928 
23d0ffd48006
plain value Keywords.keywords, which might be used outside theory for bootstrap purposes;
 wenzelm parents: 
58919diff
changeset | 139 | Keyword.is_literal keywords s) ? quote | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 140 | end | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 141 | |
| 52031 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 blanchet parents: 
51209diff
changeset | 142 | fun string_of_ext_time (plus, time) = | 
| 58081 
aa239fee063a
show microseconds as well (useful when playing with Isar proofs)
 blanchet parents: 
57728diff
changeset | 143 | let val us = Time.toMicroseconds time in | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 144 | (if plus then "> " else "") ^ | 
| 58088 | 145 | (if us < 1000 then string_of_real (Real.fromInt (us div 100) / 10.0) ^ " ms" | 
| 58081 
aa239fee063a
show microseconds as well (useful when playing with Isar proofs)
 blanchet parents: 
57728diff
changeset | 146 | else if us < 1000000 then signed_string_of_int (us div 1000) ^ " ms" | 
| 58088 | 147 | else string_of_real (Real.fromInt (us div 100000) / 10.0) ^ " s") | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 148 | end | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 149 | |
| 52031 
9a9238342963
tuning -- renamed '_from_' to '_of_' in Sledgehammer
 blanchet parents: 
51209diff
changeset | 150 | val string_of_time = string_of_ext_time o pair false | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 151 | |
| 47150 | 152 | fun type_instance thy T T' = Sign.typ_instance thy (T, T') | 
| 153 | fun type_generalization thy T T' = Sign.typ_instance thy (T', T) | |
| 48247 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 154 | |
| 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 155 | fun type_intersect _ (TVar _) _ = true | 
| 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 156 | | type_intersect _ _ (TVar _) = true | 
| 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 157 | | type_intersect thy T T' = | 
| 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 158 | let | 
| 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 159 | val tvars = Term.add_tvar_namesT T [] | 
| 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 160 | val tvars' = Term.add_tvar_namesT T' [] | 
| 50968 
3686bc0d4df2
pass correct index to "Sign.typ_unify" -- this is important to avoid what appears to be an infinite loop in the unifier
 blanchet parents: 
50239diff
changeset | 161 | val maxidx' = maxidx_of_typ T' | 
| 48247 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 162 | val T = | 
| 50968 
3686bc0d4df2
pass correct index to "Sign.typ_unify" -- this is important to avoid what appears to be an infinite loop in the unifier
 blanchet parents: 
50239diff
changeset | 163 | T |> exists (member (op =) tvars') tvars ? Logic.incr_tvar (maxidx' + 1) | 
| 
3686bc0d4df2
pass correct index to "Sign.typ_unify" -- this is important to avoid what appears to be an infinite loop in the unifier
 blanchet parents: 
50239diff
changeset | 164 | val maxidx = Integer.max (maxidx_of_typ T) maxidx' | 
| 
3686bc0d4df2
pass correct index to "Sign.typ_unify" -- this is important to avoid what appears to be an infinite loop in the unifier
 blanchet parents: 
50239diff
changeset | 165 | in can (Sign.typ_unify thy (T, T')) (Vartab.empty, maxidx) end | 
| 48247 
8f37d2ddabc8
optimized type intersection, hoping this will reduce the number of sudden Interrupts in the "incr_tvar" code
 blanchet parents: 
48238diff
changeset | 166 | |
| 47150 | 167 | val type_equiv = Sign.typ_equiv | 
| 44399 | 168 | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 169 | fun varify_type ctxt T = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 170 |   Variable.polymorphic_types ctxt [Const (@{const_name undefined}, T)]
 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 171 | |> snd |> the_single |> dest_Const |> snd | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 172 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 173 | (* TODO: use "Term_Subst.instantiateT" instead? *) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 174 | fun instantiate_type thy T1 T1' T2 = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 175 | Same.commit (Envir.subst_type_same | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 176 | (Sign.typ_match thy (T1, T1') Vartab.empty)) T2 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 177 |   handle Type.TYPE_MATCH => raise TYPE ("instantiate_type", [T1, T1'], [])
 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 178 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 179 | fun varify_and_instantiate_type ctxt T1 T1' T2 = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 180 | let val thy = Proof_Context.theory_of ctxt in | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 181 | instantiate_type thy (varify_type ctxt T1) T1' (varify_type ctxt T2) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 182 | end | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 183 | |
| 54554 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 184 | fun free_constructors_of ctxt (Type (s, Ts)) = | 
| 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 185 | (case Ctr_Sugar.ctr_sugar_of ctxt s of | 
| 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 186 |       SOME {ctrs, ...} => map_filter (try dest_Const o Ctr_Sugar.mk_ctr Ts) ctrs
 | 
| 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 187 | | NONE => []) | 
| 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 188 | | free_constructors_of _ _ = [] | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 189 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 190 | (* Similar to "Nitpick_HOL.bounded_exact_card_of_type". | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 191 | 0 means infinite type, 1 means singleton type (e.g., "unit"), and 2 means | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 192 | cardinality 2 or more. The specified default cardinality is returned if the | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 193 | cardinality of the type can't be determined. *) | 
| 44500 | 194 | fun tiny_card_of_type ctxt sound assigns default_card T = | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 195 | let | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 196 | val thy = Proof_Context.theory_of ctxt | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 197 | val max = 2 (* 1 would be too small for the "fun" case *) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 198 | fun aux slack avoid T = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 199 | if member (op =) avoid T then | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 200 | 0 | 
| 47150 | 201 | else case AList.lookup (type_equiv thy) assigns T of | 
| 44393 | 202 | SOME k => k | 
| 203 | | NONE => | |
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 204 | case T of | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 205 |           Type (@{type_name fun}, [T1, T2]) =>
 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 206 | (case (aux slack avoid T1, aux slack avoid T2) of | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 207 | (k, 1) => if slack andalso k = 0 then 0 else 1 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 208 | | (0, _) => 0 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 209 | | (_, 0) => 0 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 210 | | (k1, k2) => | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 211 | if k1 >= max orelse k2 >= max then max | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 212 | else Int.min (max, Integer.pow k2 k1)) | 
| 48230 
0feb93dfb268
gracefully compute cardinality of sets (to avoid type protectors)
 blanchet parents: 
47991diff
changeset | 213 |         | Type (@{type_name set}, [T']) => aux slack avoid (T' --> @{typ bool})
 | 
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 214 |         | @{typ prop} => 2
 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 215 |         | @{typ bool} => 2 (* optimization *)
 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 216 |         | @{typ nat} => 0 (* optimization *)
 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 217 |         | Type ("Int.int", []) => 0 (* optimization *)
 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 218 | | Type (s, _) => | 
| 54554 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 219 | (case free_constructors_of ctxt T of | 
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 220 | constrs as _ :: _ => | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 221 | let | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 222 | val constr_cards = | 
| 54554 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 223 | map (Integer.prod o map (aux slack (T :: avoid)) o binder_types o snd) constrs | 
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 224 | in | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 225 | if exists (curry (op =) 0) constr_cards then 0 | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 226 | else Int.min (max, Integer.sum constr_cards) | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 227 | end | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 228 | | [] => | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 229 | case Typedef.get_info ctxt s of | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 230 |                ({abs_type, rep_type, ...}, _) :: _ =>
 | 
| 45299 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 231 | if not sound then | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 232 | (* We cheat here by assuming that typedef types are infinite if | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 233 | their underlying type is infinite. This is unsound in | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 234 | general but it's hard to think of a realistic example where | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 235 | this would not be the case. We are also slack with | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 236 | representation types: If a representation type has the form | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 237 | "sigma => tau", we consider it enough to check "sigma" for | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 238 | infiniteness. *) | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 239 | (case varify_and_instantiate_type ctxt | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 240 | (Logic.varifyT_global abs_type) T | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 241 | (Logic.varifyT_global rep_type) | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 242 | |> aux true avoid of | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 243 | 0 => 0 | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 244 | | 1 => 1 | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 245 | | _ => default_card) | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 246 | else | 
| 
ee584ff987c3
check "sound" flag before doing something unsound...
 blanchet parents: 
44935diff
changeset | 247 | default_card | 
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 248 | | [] => default_card) | 
| 54554 
b8d0d8407c3b
eliminated Sledgehammer's dependency on old-style datatypes
 blanchet parents: 
53800diff
changeset | 249 | | TFree _ => | 
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 250 | (* Very slightly unsound: Type variables are assumed not to be | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 251 | constrained to cardinality 1. (In practice, the user would most | 
| 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 252 | likely have used "unit" directly anyway.) *) | 
| 44500 | 253 | if not sound andalso default_card = 1 then 2 else default_card | 
| 44392 
6750b4297691
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
 blanchet parents: 
43864diff
changeset | 254 | | TVar _ => default_card | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 255 | in Int.min (max, aux false [] T) end | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 256 | |
| 44500 | 257 | fun is_type_surely_finite ctxt T = tiny_card_of_type ctxt true [] 0 T <> 0 | 
| 258 | fun is_type_surely_infinite ctxt sound infinite_Ts T = | |
| 259 | tiny_card_of_type ctxt sound (map (rpair 0) infinite_Ts) 1 T = 0 | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 260 | |
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 261 | (* Simple simplifications to ensure that sort annotations don't leave a trail of | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 262 | spurious "True"s. *) | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 263 | fun s_not (Const (@{const_name All}, T) $ Abs (s, T', t')) =
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 264 |     Const (@{const_name Ex}, T) $ Abs (s, T', s_not t')
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 265 |   | s_not (Const (@{const_name Ex}, T) $ Abs (s, T', t')) =
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 266 |     Const (@{const_name All}, T) $ Abs (s, T', s_not t')
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 267 |   | s_not (@{const HOL.implies} $ t1 $ t2) = @{const HOL.conj} $ t1 $ s_not t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 268 |   | s_not (@{const HOL.conj} $ t1 $ t2) =
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 269 |     @{const HOL.disj} $ s_not t1 $ s_not t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 270 |   | s_not (@{const HOL.disj} $ t1 $ t2) =
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 271 |     @{const HOL.conj} $ s_not t1 $ s_not t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 272 |   | s_not (@{const False}) = @{const True}
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 273 |   | s_not (@{const True}) = @{const False}
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 274 |   | s_not (@{const Not} $ t) = t
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 275 |   | s_not t = @{const Not} $ t
 | 
| 54758 | 276 | |
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 277 | fun s_conj (@{const True}, t2) = t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 278 |   | s_conj (t1, @{const True}) = t1
 | 
| 51209 | 279 |   | s_conj (@{const False}, _) = @{const False}
 | 
| 280 |   | s_conj (_, @{const False}) = @{const False}
 | |
| 51197 | 281 | | s_conj (t1, t2) = if t1 aconv t2 then t1 else HOLogic.mk_conj (t1, t2) | 
| 54758 | 282 | |
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 283 | fun s_disj (@{const False}, t2) = t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 284 |   | s_disj (t1, @{const False}) = t1
 | 
| 51209 | 285 |   | s_disj (@{const True}, _) = @{const True}
 | 
| 286 |   | s_disj (_, @{const True}) = @{const True}
 | |
| 51197 | 287 | | s_disj (t1, t2) = if t1 aconv t2 then t1 else HOLogic.mk_disj (t1, t2) | 
| 54757 
4960647932ec
use 'prop' rather than 'bool' systematically in Isar reconstruction code
 blanchet parents: 
54554diff
changeset | 288 | |
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 289 | fun s_imp (@{const True}, t2) = t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 290 |   | s_imp (t1, @{const False}) = s_not t1
 | 
| 51209 | 291 |   | s_imp (@{const False}, _) = @{const True}
 | 
| 292 |   | s_imp (_, @{const True}) = @{const True}
 | |
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 293 | | s_imp p = HOLogic.mk_imp p | 
| 54757 
4960647932ec
use 'prop' rather than 'bool' systematically in Isar reconstruction code
 blanchet parents: 
54554diff
changeset | 294 | |
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 295 | fun s_iff (@{const True}, t2) = t2
 | 
| 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 296 |   | s_iff (t1, @{const True}) = t1
 | 
| 51209 | 297 |   | s_iff (@{const False}, t2) = s_not t2
 | 
| 298 |   | s_iff (t1, @{const False}) = s_not t1
 | |
| 56126 | 299 |   | s_iff (t1, t2) = if t1 aconv t2 then @{const True} else HOLogic.eq_const HOLogic.boolT $ t1 $ t2
 | 
| 43863 
a43d61270142
ensure that the lambda translation procedure is called only once with all the facts, which is necessary for soundness of lambda-lifting (freshness of new names)
 blanchet parents: 
43827diff
changeset | 300 | |
| 49983 
33e18e9916a8
use metaquantification when possible in Isar proofs
 blanchet parents: 
49982diff
changeset | 301 | fun close_form t = | 
| 
33e18e9916a8
use metaquantification when possible in Isar proofs
 blanchet parents: 
49982diff
changeset | 302 | fold (fn ((s, i), T) => fn t' => | 
| 54757 
4960647932ec
use 'prop' rather than 'bool' systematically in Isar reconstruction code
 blanchet parents: 
54554diff
changeset | 303 | Logic.all_const T $ Abs (s, T, abstract_over (Var ((s, i), T), t'))) | 
| 
4960647932ec
use 'prop' rather than 'bool' systematically in Isar reconstruction code
 blanchet parents: 
54554diff
changeset | 304 | (Term.add_vars t []) t | 
| 49983 
33e18e9916a8
use metaquantification when possible in Isar proofs
 blanchet parents: 
49982diff
changeset | 305 | |
| 58091 | 306 | val hol_close_form_prefix = "ATP." | 
| 46385 
0ccf458a3633
third attempt at lambda lifting that works for both Sledgehammer and Metis (cf. dce6c3a460a9)
 blanchet parents: 
45896diff
changeset | 307 | |
| 49982 | 308 | fun hol_close_form t = | 
| 45570 
6d95a66cce00
pull variables (Var) out of lambdas, so that the Isabelle theorems closely mirror the Metis lambda-lifted ones
 blanchet parents: 
45511diff
changeset | 309 | fold (fn ((s, i), T) => fn t' => | 
| 45511 
9b0f8ca4388e
continued implementation of lambda-lifting in Metis
 blanchet parents: 
45299diff
changeset | 310 | HOLogic.all_const T | 
| 49982 | 311 | $ Abs (hol_close_form_prefix ^ s, T, | 
| 46385 
0ccf458a3633
third attempt at lambda lifting that works for both Sledgehammer and Metis (cf. dce6c3a460a9)
 blanchet parents: 
45896diff
changeset | 312 | abstract_over (Var ((s, i), T), t'))) | 
| 43864 
58a7b3fdc193
fixed lambda-liftg: must ensure the formulas are in close form
 blanchet parents: 
43863diff
changeset | 313 | (Term.add_vars t []) t | 
| 
58a7b3fdc193
fixed lambda-liftg: must ensure the formulas are in close form
 blanchet parents: 
43863diff
changeset | 314 | |
| 49982 | 315 | fun hol_open_form unprefix | 
| 316 |       (t as Const (@{const_name All}, _) $ Abs (s, T, t')) =
 | |
| 47718 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 317 | (case try unprefix s of | 
| 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 318 | SOME s => | 
| 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 319 | let | 
| 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 320 | val names = Name.make_context (map fst (Term.add_var_names t' [])) | 
| 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 321 | val (s, _) = Name.variant s names | 
| 49982 | 322 | in hol_open_form unprefix (subst_bound (Var ((s, 0), T), t')) end | 
| 47718 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 323 | | NONE => t) | 
| 49982 | 324 | | hol_open_form _ t = t | 
| 47718 
39229c760636
smoother handling of conjecture, so that its Skolem constants get displayed in countermodels
 blanchet parents: 
47715diff
changeset | 325 | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 326 | fun eta_expand _ t 0 = t | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 327 | | eta_expand Ts (Abs (s, T, t')) n = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 328 | Abs (s, T, eta_expand (T :: Ts) t' (n - 1)) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 329 | | eta_expand Ts t n = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 330 |     fold_rev (fn T => fn t' => Abs ("x" ^ nat_subscript n, T, t'))
 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 331 | (List.take (binder_types (fastype_of1 (Ts, t)), n)) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 332 | (list_comb (incr_boundvars n t, map Bound (n - 1 downto 0))) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 333 | |
| 59632 | 334 | fun cong_extensionalize_term ctxt t = | 
| 47954 
aada9fd08b58
make higher-order goals more first-order via extensionality
 blanchet parents: 
47953diff
changeset | 335 |   if exists_Const (fn (s, _) => s = @{const_name Not}) t then
 | 
| 59632 | 336 | t |> Skip_Proof.make_thm (Proof_Context.theory_of ctxt) | 
| 337 | |> Meson.cong_extensionalize_thm ctxt | |
| 59582 | 338 | |> Thm.prop_of | 
| 47954 
aada9fd08b58
make higher-order goals more first-order via extensionality
 blanchet parents: 
47953diff
changeset | 339 | else | 
| 
aada9fd08b58
make higher-order goals more first-order via extensionality
 blanchet parents: 
47953diff
changeset | 340 | t | 
| 
aada9fd08b58
make higher-order goals more first-order via extensionality
 blanchet parents: 
47953diff
changeset | 341 | |
| 47715 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 342 | fun is_fun_equality (@{const_name HOL.eq},
 | 
| 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 343 |                      Type (_, [Type (@{type_name fun}, _), _])) = true
 | 
| 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 344 | | is_fun_equality _ = false | 
| 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 345 | |
| 47953 
a2c3706c4cb1
added "ext_cong_neq" lemma (not used yet); tuning
 blanchet parents: 
47718diff
changeset | 346 | fun abs_extensionalize_term ctxt t = | 
| 47715 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 347 | if exists_Const is_fun_equality t then | 
| 59632 | 348 | t |> Thm.cterm_of ctxt |> Meson.abs_extensionalize_conv ctxt | 
| 349 | |> Thm.prop_of |> Logic.dest_equals |> snd | |
| 47715 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 350 | else | 
| 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 351 | t | 
| 
04400144c6fc
handle TPTP definitions as definitions in Nitpick rather than as axioms
 blanchet parents: 
47150diff
changeset | 352 | |
| 47991 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 353 | fun unextensionalize_def t = | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 354 | case t of | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 355 |     @{const Trueprop} $ (Const (@{const_name HOL.eq}, _) $ lhs $ rhs) =>
 | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 356 | (case strip_comb lhs of | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 357 | (c as Const (_, T), args) => | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 358 | if forall is_Var args andalso not (has_duplicates (op =) args) then | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 359 |          @{const Trueprop}
 | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 360 |          $ (Const (@{const_name HOL.eq}, T --> T --> @{typ bool})
 | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 361 | $ c $ fold_rev lambda args rhs) | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 362 | else | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 363 | t | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 364 | | _ => t) | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 365 | | _ => t | 
| 
3eb598b044ad
make Nitpick's handling of definitions more robust in the face of formulas that don't have the expected format (needed for soundness, cf. RNG100+1)
 blanchet parents: 
47954diff
changeset | 366 | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 367 | (* Converts an elim-rule into an equivalent theorem that does not have the | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 368 | predicate variable. Leaves other theorems unchanged. We simply instantiate | 
| 44460 | 369 | the conclusion variable to "False". (Cf. "transform_elim_theorem" in | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 370 | "Meson_Clausify".) *) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 371 | fun transform_elim_prop t = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 372 | case Logic.strip_imp_concl t of | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 373 |     @{const Trueprop} $ Var (z, @{typ bool}) =>
 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 374 |     subst_Vars [(z, @{const False})] t
 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 375 |   | Var (z, @{typ prop}) => subst_Vars [(z, @{prop False})] t
 | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 376 | | _ => t | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 377 | |
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 378 | fun specialize_type thy (s, T) t = | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 379 | let | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 380 | fun subst_for (Const (s', T')) = | 
| 61769 | 381 | if s = s' then | 
| 382 | SOME (Sign.typ_match thy (T', T) Vartab.empty) | |
| 383 | handle Type.TYPE_MATCH => NONE | |
| 384 | else | |
| 385 | NONE | |
| 386 | | subst_for (t1 $ t2) = (case subst_for t1 of SOME x => SOME x | NONE => subst_for t2) | |
| 387 | | subst_for (Abs (_, _, t')) = subst_for t' | |
| 388 | | subst_for _ = NONE | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 389 | in | 
| 61769 | 390 | (case subst_for t of | 
| 61770 | 391 | SOME subst => Envir.subst_term_types subst t | 
| 61769 | 392 | | NONE => raise Type.TYPE_MATCH) | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 393 | end | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 394 | |
| 52125 
ac7830871177
improved handling of free variables' types in Isar proofs
 blanchet parents: 
52077diff
changeset | 395 | fun strip_subgoal goal i ctxt = | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 396 | let | 
| 52196 
2281f33e8da6
redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
 blanchet parents: 
52125diff
changeset | 397 | val (t, (frees, params)) = | 
| 59582 | 398 | Logic.goal_params (Thm.prop_of goal) i | 
| 52196 
2281f33e8da6
redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
 blanchet parents: 
52125diff
changeset | 399 | ||> (map dest_Free #> Variable.variant_frees ctxt [] #> `(map Free)) | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 400 | val hyp_ts = t |> Logic.strip_assums_hyp |> map (curry subst_bounds frees) | 
| 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 401 | val concl_t = t |> Logic.strip_assums_concl |> curry subst_bounds frees | 
| 52196 
2281f33e8da6
redid rac7830871177 to avoid duplicate fixed variable (e.g. lemma "P (a::nat)" proof - have "!!a::int. Q a" sledgehammer [e])
 blanchet parents: 
52125diff
changeset | 402 | in (rev params, hyp_ts, concl_t) end | 
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 403 | |
| 57541 | 404 | fun extract_lambda_def dest_head (Const (@{const_name HOL.eq}, _) $ t $ u) =
 | 
| 405 | let val (head, args) = strip_comb t in | |
| 406 | (head |> dest_head |> fst, | |
| 407 | fold_rev (fn t as Var ((s, _), T) => | |
| 408 | (fn u => Abs (s, T, abstract_over (t, u))) | |
| 409 | | _ => raise Fail "expected \"Var\"") args u) | |
| 410 | end | |
| 411 | | extract_lambda_def _ _ = raise Fail "malformed lifted lambda" | |
| 412 | ||
| 56104 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 413 | fun short_thm_name ctxt th = | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 414 | let | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 415 | val long = Thm.get_name_hint th | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 416 | val short = Long_Name.base_name long | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 417 | in | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 418 | if Thm.eq_thm_prop (th, singleton (Attrib.eval_thms ctxt) (Facts.named short, [])) then short | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 419 | else long | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 420 | end | 
| 
fd6e132ee4fb
correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
 blanchet parents: 
54768diff
changeset | 421 | |
| 43085 
0a2f5b86bdd7
first step in sharing more code between ATP and Metis translation
 blanchet parents: diff
changeset | 422 | end; |