author | wenzelm |
Tue, 09 Apr 2013 21:14:00 +0200 | |
changeset 51665 | cba83c9f72b9 |
parent 47909 | 5f1afeebafbc |
child 51685 | 385ef6706252 |
permissions | -rw-r--r-- |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1 |
(* Title: HOL/Tools/Nitpick/nitpick_preproc.ML |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
2 |
Author: Jasmin Blanchette, TU Muenchen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
3 |
Copyright 2008, 2009, 2010 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
4 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
5 |
Nitpick's HOL preprocessor. |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
6 |
*) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
7 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
8 |
signature NITPICK_PREPROC = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
9 |
sig |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
10 |
type hol_context = Nitpick_HOL.hol_context |
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
11 |
val preprocess_formulas : |
41052
3db267a01c1d
remove the "fin_fun" optimization in Nitpick -- it was always a hack and didn't help much
blanchet
parents:
41001
diff
changeset
|
12 |
hol_context -> term list -> term |
41803
ef13e3b7cbaf
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet
parents:
41793
diff
changeset
|
13 |
-> term list * term list * term list * bool * bool * bool |
35866
513074557e06
move the Sledgehammer Isar commands together into one file;
blanchet
parents:
35807
diff
changeset
|
14 |
end; |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
15 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
16 |
structure Nitpick_Preproc : NITPICK_PREPROC = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
17 |
struct |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
18 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
19 |
open Nitpick_Util |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
20 |
open Nitpick_HOL |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35408
diff
changeset
|
21 |
open Nitpick_Mono |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
22 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
23 |
fun is_positive_existential polar quant_s = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
24 |
(polar = Pos andalso quant_s = @{const_name Ex}) orelse |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
25 |
(polar = Neg andalso quant_s <> @{const_name Ex}) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
26 |
|
37271 | 27 |
val is_descr = |
39360
cdf2c3341422
eliminate more clutter related to "fast_descrs" optimization
blanchet
parents:
39359
diff
changeset
|
28 |
member (op =) [@{const_name The}, @{const_name Eps}, @{const_name safe_The}] |
37271 | 29 |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
30 |
(** Binary coding of integers **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
31 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
32 |
(* If a formula contains a numeral whose absolute value is more than this |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
33 |
threshold, the unary coding is likely not to work well and we prefer the |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
34 |
binary coding. *) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
35 |
val binary_int_threshold = 3 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
36 |
|
35718 | 37 |
val may_use_binary_ints = |
38 |
let |
|
39 |
fun aux def (Const (@{const_name "=="}, _) $ t1 $ t2) = |
|
40 |
aux def t1 andalso aux false t2 |
|
41 |
| aux def (@{const "==>"} $ t1 $ t2) = aux false t1 andalso aux def t2 |
|
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
42 |
| aux def (Const (@{const_name HOL.eq}, _) $ t1 $ t2) = |
35718 | 43 |
aux def t1 andalso aux false t2 |
38786
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
44 |
| aux def (@{const HOL.implies} $ t1 $ t2) = aux false t1 andalso aux def t2 |
35718 | 45 |
| aux def (t1 $ t2) = aux def t1 andalso aux def t2 |
46 |
| aux def (t as Const (s, _)) = |
|
47 |
(not def orelse t <> @{const Suc}) andalso |
|
47909
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
48 |
not (member (op =) |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
49 |
[@{const_name Nitpick.Abs_Frac}, @{const_name Nitpick.Rep_Frac}, |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
50 |
@{const_name Nitpick.nat_gcd}, @{const_name Nitpick.nat_lcm}, |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
51 |
@{const_name Nitpick.Frac}, @{const_name Nitpick.norm_frac}] s) |
35718 | 52 |
| aux def (Abs (_, _, t')) = aux def t' |
53 |
| aux _ _ = true |
|
54 |
in aux end |
|
55 |
val should_use_binary_ints = |
|
56 |
let |
|
57 |
fun aux (t1 $ t2) = aux t1 orelse aux t2 |
|
58 |
| aux (Const (s, T)) = |
|
59 |
((s = @{const_name times} orelse s = @{const_name div}) andalso |
|
60 |
is_integer_type (body_type T)) orelse |
|
61 |
(String.isPrefix numeral_prefix s andalso |
|
62 |
let val n = the (Int.fromString (unprefix numeral_prefix s)) in |
|
63 |
n < ~ binary_int_threshold orelse n > binary_int_threshold |
|
64 |
end) |
|
65 |
| aux (Abs (_, _, t')) = aux t' |
|
66 |
| aux _ = false |
|
67 |
in aux end |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
68 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
69 |
(** Uncurrying **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
70 |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
71 |
fun add_to_uncurry_table ctxt t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
72 |
let |
42361 | 73 |
val thy = Proof_Context.theory_of ctxt |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
74 |
fun aux (t1 $ t2) args table = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
75 |
let val table = aux t2 [] table in aux t1 (t2 :: args) table end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
76 |
| aux (Abs (_, _, t')) _ table = aux t' [] table |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
77 |
| aux (t as Const (x as (s, _))) args table = |
39359 | 78 |
if is_built_in_const thy [(NONE, true)] x orelse |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
79 |
is_constr_like ctxt x orelse |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
80 |
is_sel s orelse s = @{const_name Sigma} then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
81 |
table |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
82 |
else |
36384 | 83 |
Termtab.map_default (t, 65536) (Integer.min (length args)) table |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
84 |
| aux _ _ table = table |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
85 |
in aux t [] end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
86 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
87 |
fun uncurry_prefix_for k j = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
88 |
uncurry_prefix ^ string_of_int k ^ "@" ^ string_of_int j ^ name_sep |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
89 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
90 |
fun uncurry_term table t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
91 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
92 |
fun aux (t1 $ t2) args = aux t1 (aux t2 [] :: args) |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
93 |
| aux (Abs (s, T, t')) args = s_betapplys [] (Abs (s, T, aux t' []), args) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
94 |
| aux (t as Const (s, T)) args = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
95 |
(case Termtab.lookup table t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
96 |
SOME n => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
97 |
if n >= 2 then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
98 |
let |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
99 |
val arg_Ts = strip_n_binders n T |> fst |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
100 |
val j = |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
101 |
if is_iterator_type (hd arg_Ts) then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
102 |
1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
103 |
else case find_index (not_equal bool_T) arg_Ts of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
104 |
~1 => n |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
105 |
| j => j |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
106 |
val ((before_args, tuple_args), after_args) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
107 |
args |> chop n |>> chop j |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
108 |
val ((before_arg_Ts, tuple_arg_Ts), rest_T) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
109 |
T |> strip_n_binders n |>> chop j |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
110 |
val tuple_T = HOLogic.mk_tupleT tuple_arg_Ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
111 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
112 |
if n - j < 2 then |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
113 |
s_betapplys [] (t, args) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
114 |
else |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
115 |
s_betapplys [] |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
116 |
(Const (uncurry_prefix_for (n - j) j ^ s, |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
117 |
before_arg_Ts ---> tuple_T --> rest_T), |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
118 |
before_args @ [mk_flat_tuple tuple_T tuple_args] @ |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
119 |
after_args) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
120 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
121 |
else |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
122 |
s_betapplys [] (t, args) |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
123 |
| NONE => s_betapplys [] (t, args)) |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
124 |
| aux t args = s_betapplys [] (t, args) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
125 |
in aux t [] end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
126 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
127 |
(** Boxing **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
128 |
|
39359 | 129 |
fun box_fun_and_pair_in_term (hol_ctxt as {ctxt, thy, stds, ...}) def orig_t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
130 |
let |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35408
diff
changeset
|
131 |
fun box_relational_operator_type (Type (@{type_name fun}, Ts)) = |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35408
diff
changeset
|
132 |
Type (@{type_name fun}, map box_relational_operator_type Ts) |
38190
b02e204b613a
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
blanchet
parents:
38170
diff
changeset
|
133 |
| box_relational_operator_type (Type (@{type_name prod}, Ts)) = |
b02e204b613a
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
blanchet
parents:
38170
diff
changeset
|
134 |
Type (@{type_name prod}, map (box_type hol_ctxt InPair) Ts) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
135 |
| box_relational_operator_type T = T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
136 |
fun add_boxed_types_for_var (z as (_, T)) (T', t') = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
137 |
case t' of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
138 |
Var z' => z' = z ? insert (op =) T' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
139 |
| Const (@{const_name Pair}, _) $ t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
140 |
(case T' of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
141 |
Type (_, [T1, T2]) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
142 |
fold (add_boxed_types_for_var z) [(T1, t1), (T2, t2)] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
143 |
| _ => raise TYPE ("Nitpick_Preproc.box_fun_and_pair_in_term.\ |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
144 |
\add_boxed_types_for_var", [T'], [])) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
145 |
| _ => exists_subterm (curry (op =) (Var z)) t' ? insert (op =) T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
146 |
fun box_var_in_def new_Ts old_Ts t (z as (_, T)) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
147 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
148 |
@{const Trueprop} $ t1 => box_var_in_def new_Ts old_Ts t1 z |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
149 |
| Const (s0, _) $ t1 $ _ => |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
150 |
if s0 = @{const_name "=="} orelse s0 = @{const_name HOL.eq} then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
151 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
152 |
val (t', args) = strip_comb t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
153 |
val T' = fastype_of1 (new_Ts, do_term new_Ts old_Ts Neut t') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
154 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
155 |
case fold (add_boxed_types_for_var z) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
156 |
(fst (strip_n_binders (length args) T') ~~ args) [] of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
157 |
[T''] => T'' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
158 |
| _ => T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
159 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
160 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
161 |
T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
162 |
| _ => T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
163 |
and do_quantifier new_Ts old_Ts polar quant_s quant_T abs_s abs_T t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
164 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
165 |
val abs_T' = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
166 |
if polar = Neut orelse is_positive_existential polar quant_s then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
167 |
box_type hol_ctxt InFunLHS abs_T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
168 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
169 |
abs_T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
170 |
val body_T = body_type quant_T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
171 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
172 |
Const (quant_s, (abs_T' --> body_T) --> body_T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
173 |
$ Abs (abs_s, abs_T', |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
174 |
t |> do_term (abs_T' :: new_Ts) (abs_T :: old_Ts) polar) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
175 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
176 |
and do_equals new_Ts old_Ts s0 T0 t1 t2 = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
177 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
178 |
val (t1, t2) = pairself (do_term new_Ts old_Ts Neut) (t1, t2) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
179 |
val (T1, T2) = pairself (curry fastype_of1 new_Ts) (t1, t2) |
37704
c6161bee8486
adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
blanchet
parents:
37678
diff
changeset
|
180 |
val T = if def then T1 |
c6161bee8486
adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
blanchet
parents:
37678
diff
changeset
|
181 |
else [T1, T2] |> sort (int_ord o pairself size_of_typ) |> hd |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
182 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
183 |
list_comb (Const (s0, T --> T --> body_type T0), |
35384 | 184 |
map2 (coerce_term hol_ctxt new_Ts T) [T1, T2] [t1, t2]) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
185 |
end |
37271 | 186 |
and do_descr s T = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
187 |
let val T1 = box_type hol_ctxt InFunLHS (range_type T) in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
188 |
Const (s, (T1 --> bool_T) --> T1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
189 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
190 |
and do_term new_Ts old_Ts polar t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
191 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
192 |
Const (s0 as @{const_name all}, T0) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
193 |
do_quantifier new_Ts old_Ts polar s0 T0 s1 T1 t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
194 |
| Const (s0 as @{const_name "=="}, T0) $ t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
195 |
do_equals new_Ts old_Ts s0 T0 t1 t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
196 |
| @{const "==>"} $ t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
197 |
@{const "==>"} $ do_term new_Ts old_Ts (flip_polarity polar) t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
198 |
$ do_term new_Ts old_Ts polar t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
199 |
| @{const Pure.conjunction} $ t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
200 |
@{const Pure.conjunction} $ do_term new_Ts old_Ts polar t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
201 |
$ do_term new_Ts old_Ts polar t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
202 |
| @{const Trueprop} $ t1 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
203 |
@{const Trueprop} $ do_term new_Ts old_Ts polar t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
204 |
| @{const Not} $ t1 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
205 |
@{const Not} $ do_term new_Ts old_Ts (flip_polarity polar) t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
206 |
| Const (s0 as @{const_name All}, T0) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
207 |
do_quantifier new_Ts old_Ts polar s0 T0 s1 T1 t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
208 |
| Const (s0 as @{const_name Ex}, T0) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
209 |
do_quantifier new_Ts old_Ts polar s0 T0 s1 T1 t1 |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
210 |
| Const (s0 as @{const_name HOL.eq}, T0) $ t1 $ t2 => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
211 |
do_equals new_Ts old_Ts s0 T0 t1 t2 |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
212 |
| @{const HOL.conj} $ t1 $ t2 => |
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
213 |
@{const HOL.conj} $ do_term new_Ts old_Ts polar t1 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
214 |
$ do_term new_Ts old_Ts polar t2 |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
215 |
| @{const HOL.disj} $ t1 $ t2 => |
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
216 |
@{const HOL.disj} $ do_term new_Ts old_Ts polar t1 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
217 |
$ do_term new_Ts old_Ts polar t2 |
38786
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
218 |
| @{const HOL.implies} $ t1 $ t2 => |
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
219 |
@{const HOL.implies} $ do_term new_Ts old_Ts (flip_polarity polar) t1 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
220 |
$ do_term new_Ts old_Ts polar t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
221 |
| Const (x as (s, T)) => |
37271 | 222 |
if is_descr s then |
223 |
do_descr s T |
|
224 |
else |
|
225 |
Const (s, if s = @{const_name converse} orelse |
|
226 |
s = @{const_name trancl} then |
|
227 |
box_relational_operator_type T |
|
228 |
else if String.isPrefix quot_normal_prefix s then |
|
229 |
let val T' = box_type hol_ctxt InFunLHS (domain_type T) in |
|
230 |
T' --> T' |
|
231 |
end |
|
39359 | 232 |
else if is_built_in_const thy stds x orelse |
37271 | 233 |
s = @{const_name Sigma} then |
234 |
T |
|
235 |
else if is_constr_like ctxt x then |
|
236 |
box_type hol_ctxt InConstr T |
|
237 |
else if is_sel s orelse is_rep_fun ctxt x then |
|
238 |
box_type hol_ctxt InSel T |
|
239 |
else |
|
240 |
box_type hol_ctxt InExpr T) |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
241 |
| t1 $ Abs (s, T, t2') => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
242 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
243 |
val t1 = do_term new_Ts old_Ts Neut t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
244 |
val T1 = fastype_of1 (new_Ts, t1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
245 |
val (s1, Ts1) = dest_Type T1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
246 |
val T' = hd (snd (dest_Type (hd Ts1))) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
247 |
val t2 = Abs (s, T', do_term (T' :: new_Ts) (T :: old_Ts) Neut t2') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
248 |
val T2 = fastype_of1 (new_Ts, t2) |
35384 | 249 |
val t2 = coerce_term hol_ctxt new_Ts (hd Ts1) T2 t2 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
250 |
in |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
251 |
s_betapply new_Ts (if s1 = @{type_name fun} then |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
252 |
t1 |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
253 |
else |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
254 |
select_nth_constr_arg ctxt stds |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
255 |
(@{const_name FunBox}, |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
256 |
Type (@{type_name fun}, Ts1) --> T1) t1 0 |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
257 |
(Type (@{type_name fun}, Ts1)), t2) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
258 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
259 |
| t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
260 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
261 |
val t1 = do_term new_Ts old_Ts Neut t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
262 |
val T1 = fastype_of1 (new_Ts, t1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
263 |
val (s1, Ts1) = dest_Type T1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
264 |
val t2 = do_term new_Ts old_Ts Neut t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
265 |
val T2 = fastype_of1 (new_Ts, t2) |
35384 | 266 |
val t2 = coerce_term hol_ctxt new_Ts (hd Ts1) T2 t2 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
267 |
in |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
268 |
s_betapply new_Ts (if s1 = @{type_name fun} then |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
269 |
t1 |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
270 |
else |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
271 |
select_nth_constr_arg ctxt stds |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
272 |
(@{const_name FunBox}, |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
273 |
Type (@{type_name fun}, Ts1) --> T1) t1 0 |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
274 |
(Type (@{type_name fun}, Ts1)), t2) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
275 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
276 |
| Free (s, T) => Free (s, box_type hol_ctxt InExpr T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
277 |
| Var (z as (x, T)) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
278 |
Var (x, if def then box_var_in_def new_Ts old_Ts orig_t z |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
279 |
else box_type hol_ctxt InExpr T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
280 |
| Bound _ => t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
281 |
| Abs (s, T, t') => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
282 |
Abs (s, T, do_term (T :: new_Ts) (T :: old_Ts) Neut t') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
283 |
in do_term [] [] Pos orig_t end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
284 |
|
46102 | 285 |
(** Destruction of set membership and comprehensions **) |
286 |
||
287 |
fun destroy_set_Collect (Const (@{const_name Set.member}, _) $ t1 |
|
288 |
$ (Const (@{const_name Collect}, _) $ t2)) = |
|
289 |
destroy_set_Collect (t2 $ t1) |
|
290 |
| destroy_set_Collect (t1 $ t2) = |
|
291 |
destroy_set_Collect t1 $ destroy_set_Collect t2 |
|
292 |
| destroy_set_Collect (Abs (s, T, t')) = Abs (s, T, destroy_set_Collect t') |
|
293 |
| destroy_set_Collect t = t |
|
294 |
||
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
295 |
(** Destruction of constructors **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
296 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
297 |
val val_var_prefix = nitpick_prefix ^ "v" |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
298 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
299 |
fun fresh_value_var Ts k n j t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
300 |
Var ((val_var_prefix ^ nat_subscript (n - j), k), fastype_of1 (Ts, t)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
301 |
|
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
302 |
fun has_heavy_bounds_or_vars Ts t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
303 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
304 |
fun aux [] = false |
46115 | 305 |
| aux [T] = is_fun_or_set_type T orelse is_pair_type T |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
306 |
| aux _ = true |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
307 |
in aux (map snd (Term.add_vars t []) @ map (nth Ts) (loose_bnos t)) end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
308 |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
309 |
fun pull_out_constr_comb ({ctxt, stds, ...} : hol_context) Ts relax k level t |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
310 |
args seen = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
311 |
let val t_comb = list_comb (t, args) in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
312 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
313 |
Const x => |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
314 |
if not relax andalso is_constr ctxt stds x andalso |
46115 | 315 |
not (is_fun_or_set_type (fastype_of1 (Ts, t_comb))) andalso |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
316 |
has_heavy_bounds_or_vars Ts t_comb andalso |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
317 |
not (loose_bvar (t_comb, level)) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
318 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
319 |
val (j, seen) = case find_index (curry (op =) t_comb) seen of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
320 |
~1 => (0, t_comb :: seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
321 |
| j => (j, seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
322 |
in (fresh_value_var Ts k (length seen) j t_comb, seen) end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
323 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
324 |
(t_comb, seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
325 |
| _ => (t_comb, seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
326 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
327 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
328 |
fun equations_for_pulled_out_constrs mk_eq Ts k seen = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
329 |
let val n = length seen in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
330 |
map2 (fn j => fn t => mk_eq (fresh_value_var Ts k n j t, t)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
331 |
(index_seq 0 n) seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
332 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
333 |
|
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
334 |
fun pull_out_universal_constrs hol_ctxt def t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
335 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
336 |
val k = maxidx_of_term t + 1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
337 |
fun do_term Ts def t args seen = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
338 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
339 |
(t0 as Const (@{const_name "=="}, _)) $ t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
340 |
do_eq_or_imp Ts true def t0 t1 t2 seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
341 |
| (t0 as @{const "==>"}) $ t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
342 |
if def then (t, []) else do_eq_or_imp Ts false def t0 t1 t2 seen |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
343 |
| (t0 as Const (@{const_name HOL.eq}, _)) $ t1 $ t2 => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
344 |
do_eq_or_imp Ts true def t0 t1 t2 seen |
38786
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
345 |
| (t0 as @{const HOL.implies}) $ t1 $ t2 => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
346 |
do_eq_or_imp Ts false def t0 t1 t2 seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
347 |
| Abs (s, T, t') => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
348 |
let val (t', seen) = do_term (T :: Ts) def t' [] seen in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
349 |
(list_comb (Abs (s, T, t'), args), seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
350 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
351 |
| t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
352 |
let val (t2, seen) = do_term Ts def t2 [] seen in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
353 |
do_term Ts def t1 (t2 :: args) seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
354 |
end |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
355 |
| _ => pull_out_constr_comb hol_ctxt Ts def k 0 t args seen |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
356 |
and do_eq_or_imp Ts eq def t0 t1 t2 seen = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
357 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
358 |
val (t2, seen) = if eq andalso def then (t2, seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
359 |
else do_term Ts false t2 [] seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
360 |
val (t1, seen) = do_term Ts false t1 [] seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
361 |
in (t0 $ t1 $ t2, seen) end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
362 |
val (concl, seen) = do_term [] def t [] [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
363 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
364 |
Logic.list_implies (equations_for_pulled_out_constrs Logic.mk_equals [] k |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
365 |
seen, concl) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
366 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
367 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
368 |
fun mk_exists v t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
369 |
HOLogic.exists_const (fastype_of v) $ lambda v (incr_boundvars 1 t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
370 |
|
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
371 |
fun pull_out_existential_constrs hol_ctxt t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
372 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
373 |
val k = maxidx_of_term t + 1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
374 |
fun aux Ts num_exists t args seen = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
375 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
376 |
(t0 as Const (@{const_name Ex}, _)) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
377 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
378 |
val (t1, seen') = aux (T1 :: Ts) (num_exists + 1) t1 [] [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
379 |
val n = length seen' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
380 |
fun vars () = map2 (fresh_value_var Ts k n) (index_seq 0 n) seen' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
381 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
382 |
(equations_for_pulled_out_constrs HOLogic.mk_eq Ts k seen' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
383 |
|> List.foldl s_conj t1 |> fold mk_exists (vars ()) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
384 |
|> curry3 Abs s1 T1 |> curry (op $) t0, seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
385 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
386 |
| t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
387 |
let val (t2, seen) = aux Ts num_exists t2 [] seen in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
388 |
aux Ts num_exists t1 (t2 :: args) seen |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
389 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
390 |
| Abs (s, T, t') => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
391 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
392 |
val (t', seen) = aux (T :: Ts) 0 t' [] (map (incr_boundvars 1) seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
393 |
in (list_comb (Abs (s, T, t'), args), map (incr_boundvars ~1) seen) end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
394 |
| _ => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
395 |
if num_exists > 0 then |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
396 |
pull_out_constr_comb hol_ctxt Ts false k num_exists t args seen |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
397 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
398 |
(list_comb (t, args), seen) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
399 |
in aux [] 0 t [] [] |> fst end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
400 |
|
41994
c567c860caf6
always destroy constructor patterns, since this seems to be always useful
blanchet
parents:
41876
diff
changeset
|
401 |
fun destroy_pulled_out_constrs (hol_ctxt as {ctxt, stds, ...}) axiom strong t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
402 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
403 |
val num_occs_of_var = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
404 |
fold_aterms (fn Var z => (fn f => fn z' => f z' |> z = z' ? Integer.add 1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
405 |
| _ => I) t (K 0) |
41793
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
406 |
fun aux Ts careful ((t0 as Const (@{const_name "=="}, _)) $ t1 $ t2) = |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
407 |
aux_eq Ts careful true t0 t1 t2 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
408 |
| aux Ts careful ((t0 as @{const "==>"}) $ t1 $ t2) = |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
409 |
t0 $ aux Ts false t1 $ aux Ts careful t2 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
410 |
| aux Ts careful ((t0 as Const (@{const_name HOL.eq}, _)) $ t1 $ t2) = |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
411 |
aux_eq Ts careful true t0 t1 t2 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
412 |
| aux Ts careful ((t0 as @{const HOL.implies}) $ t1 $ t2) = |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
413 |
t0 $ aux Ts false t1 $ aux Ts careful t2 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
414 |
| aux Ts careful (Abs (s, T, t')) = Abs (s, T, aux (T :: Ts) careful t') |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
415 |
| aux Ts careful (t1 $ t2) = aux Ts careful t1 $ aux Ts careful t2 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
416 |
| aux _ _ t = t |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
417 |
and aux_eq Ts careful pass1 t0 t1 t2 = |
41994
c567c860caf6
always destroy constructor patterns, since this seems to be always useful
blanchet
parents:
41876
diff
changeset
|
418 |
((if careful orelse |
c567c860caf6
always destroy constructor patterns, since this seems to be always useful
blanchet
parents:
41876
diff
changeset
|
419 |
not (strong orelse forall (is_constr_pattern ctxt) [t1, t2]) then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
420 |
raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
421 |
else if axiom andalso is_Var t2 andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
422 |
num_occs_of_var (dest_Var t2) = 1 then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
423 |
@{const True} |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
424 |
else case strip_comb t2 of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
425 |
(* The first case is not as general as it could be. *) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
426 |
(Const (@{const_name PairBox}, _), |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
427 |
[Const (@{const_name fst}, _) $ Var z1, |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
428 |
Const (@{const_name snd}, _) $ Var z2]) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
429 |
if z1 = z2 andalso num_occs_of_var z1 = 2 then @{const True} |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
430 |
else raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
431 |
| (Const (x as (s, T)), args) => |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
432 |
let |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
433 |
val (arg_Ts, dataT) = strip_type T |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
434 |
val n = length arg_Ts |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
435 |
in |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
436 |
if length args = n andalso |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
437 |
(is_constr ctxt stds x orelse s = @{const_name Pair} orelse |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
438 |
x = (@{const_name Suc}, nat_T --> nat_T)) andalso |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
439 |
(not careful orelse not (is_Var t1) orelse |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
440 |
String.isPrefix val_var_prefix (fst (fst (dest_Var t1)))) then |
41793
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
441 |
s_let Ts "l" (n + 1) dataT bool_T |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
442 |
(fn t1 => |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
443 |
discriminate_value hol_ctxt x t1 :: |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
444 |
map3 (sel_eq Ts x t1) (index_seq 0 n) arg_Ts args |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
445 |
|> foldr1 s_conj) t1 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
446 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
447 |
raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
448 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
449 |
| _ => raise SAME ()) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
450 |
|> body_type (type_of t0) = prop_T ? HOLogic.mk_Trueprop) |
41793
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
451 |
handle SAME () => if pass1 then aux_eq Ts careful false t0 t2 t1 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
452 |
else t0 $ aux Ts false t2 $ aux Ts false t1 |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
453 |
and sel_eq Ts x t n nth_T nth_t = |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
454 |
HOLogic.eq_const nth_T $ nth_t |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
455 |
$ select_nth_constr_arg ctxt stds x t n nth_T |
41793
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
456 |
|> aux Ts false |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
457 |
in aux [] axiom t end |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
458 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
459 |
(** Destruction of universal and existential equalities **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
460 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
461 |
fun curry_assms (@{const "==>"} $ (@{const Trueprop} |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
462 |
$ (@{const HOL.conj} $ t1 $ t2)) $ t3) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
463 |
curry_assms (Logic.list_implies ([t1, t2] |> map HOLogic.mk_Trueprop, t3)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
464 |
| curry_assms (@{const "==>"} $ t1 $ t2) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
465 |
@{const "==>"} $ curry_assms t1 $ curry_assms t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
466 |
| curry_assms t = t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
467 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
468 |
val destroy_universal_equalities = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
469 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
470 |
fun aux prems zs t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
471 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
472 |
@{const "==>"} $ t1 $ t2 => aux_implies prems zs t1 t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
473 |
| _ => Logic.list_implies (rev prems, t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
474 |
and aux_implies prems zs t1 t2 = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
475 |
case t1 of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
476 |
Const (@{const_name "=="}, _) $ Var z $ t' => aux_eq prems zs z t' t1 t2 |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
477 |
| @{const Trueprop} $ (Const (@{const_name HOL.eq}, _) $ Var z $ t') => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
478 |
aux_eq prems zs z t' t1 t2 |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
479 |
| @{const Trueprop} $ (Const (@{const_name HOL.eq}, _) $ t' $ Var z) => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
480 |
aux_eq prems zs z t' t1 t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
481 |
| _ => aux (t1 :: prems) (Term.add_vars t1 zs) t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
482 |
and aux_eq prems zs z t' t1 t2 = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
483 |
if not (member (op =) zs z) andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
484 |
not (exists_subterm (curry (op =) (Var z)) t') then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
485 |
aux prems zs (subst_free [(Var z, t')] t2) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
486 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
487 |
aux (t1 :: prems) (Term.add_vars t1 zs) t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
488 |
in aux [] [] end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
489 |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
490 |
fun find_bound_assign ctxt stds j = |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
491 |
let |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
492 |
fun do_term _ [] = NONE |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
493 |
| do_term seen (t :: ts) = |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
494 |
let |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
495 |
fun do_eq pass1 t1 t2 = |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
496 |
(if loose_bvar1 (t2, j) then |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
497 |
if pass1 then do_eq false t2 t1 else raise SAME () |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
498 |
else case t1 of |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
499 |
Bound j' => if j' = j then SOME (t2, ts @ seen) else raise SAME () |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35408
diff
changeset
|
500 |
| Const (s, Type (@{type_name fun}, [T1, T2])) $ Bound j' => |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
501 |
if j' = j andalso |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
502 |
s = nth_sel_name_for_constr_name @{const_name FunBox} 0 then |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
503 |
SOME (construct_value ctxt stds |
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
504 |
(@{const_name FunBox}, T2 --> T1) [t2], |
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
505 |
ts @ seen) |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
506 |
else |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
507 |
raise SAME () |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
508 |
| _ => raise SAME ()) |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
509 |
handle SAME () => do_term (t :: seen) ts |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
510 |
in |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
511 |
case t of |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
512 |
Const (@{const_name HOL.eq}, _) $ t1 $ t2 => do_eq true t1 t2 |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
513 |
| _ => do_term (t :: seen) ts |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
514 |
end |
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
515 |
in do_term end |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
516 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
517 |
fun subst_one_bound j arg t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
518 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
519 |
fun aux (Bound i, lev) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
520 |
if i < lev then raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
521 |
else if i = lev then incr_boundvars (lev - j) arg |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
522 |
else Bound (i - 1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
523 |
| aux (Abs (a, T, body), lev) = Abs (a, T, aux (body, lev + 1)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
524 |
| aux (f $ t, lev) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
525 |
(aux (f, lev) $ (aux (t, lev) handle SAME () => t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
526 |
handle SAME () => f $ aux (t, lev)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
527 |
| aux _ = raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
528 |
in aux (t, j) handle SAME () => t end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
529 |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
530 |
fun destroy_existential_equalities ({ctxt, stds, ...} : hol_context) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
531 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
532 |
fun kill [] [] ts = foldr1 s_conj ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
533 |
| kill (s :: ss) (T :: Ts) ts = |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
534 |
(case find_bound_assign ctxt stds (length ss) [] ts of |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
535 |
SOME (_, []) => @{const True} |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
536 |
| SOME (arg_t, ts) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
537 |
kill ss Ts (map (subst_one_bound (length ss) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
538 |
(incr_bv (~1, length ss + 1, arg_t))) ts) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
539 |
| NONE => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
540 |
Const (@{const_name Ex}, (T --> bool_T) --> bool_T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
541 |
$ Abs (s, T, kill ss Ts ts)) |
40722
441260986b63
make two copies (!) of Library.UnequalLengths coincide with ListPair.UnequalLengths;
wenzelm
parents:
39687
diff
changeset
|
542 |
| kill _ _ _ = raise ListPair.UnequalLengths |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
543 |
fun gather ss Ts (Const (@{const_name Ex}, _) $ Abs (s1, T1, t1)) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
544 |
gather (ss @ [s1]) (Ts @ [T1]) t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
545 |
| gather [] [] (Abs (s, T, t1)) = Abs (s, T, gather [] [] t1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
546 |
| gather [] [] (t1 $ t2) = gather [] [] t1 $ gather [] [] t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
547 |
| gather [] [] t = t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
548 |
| gather ss Ts t = kill ss Ts (conjuncts_of (gather [] [] t)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
549 |
in gather [] [] end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
550 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
551 |
(** Skolemization **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
552 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
553 |
fun skolem_prefix_for k j = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
554 |
skolem_prefix ^ string_of_int k ^ "@" ^ string_of_int j ^ name_sep |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
555 |
|
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
556 |
fun skolemize_term_and_more (hol_ctxt as {thy, def_tables, skolems, ...}) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
557 |
skolem_depth = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
558 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
559 |
val incrs = map (Integer.add 1) |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
560 |
fun aux ss Ts js skolemizable polar t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
561 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
562 |
fun do_quantifier quant_s quant_T abs_s abs_T t = |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
563 |
(if not (loose_bvar1 (t, 0)) then |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
564 |
aux ss Ts js skolemizable polar (incr_boundvars ~1 t) |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
565 |
else if is_positive_existential polar quant_s then |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
566 |
let |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
567 |
val j = length (!skolems) + 1 |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
568 |
in |
47754
11b4395aaf0c
remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
blanchet
parents:
47669
diff
changeset
|
569 |
if skolemizable andalso length js <= skolem_depth then |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
570 |
let |
47754
11b4395aaf0c
remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
blanchet
parents:
47669
diff
changeset
|
571 |
val sko_s = skolem_prefix_for (length js) j ^ abs_s |
11b4395aaf0c
remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
blanchet
parents:
47669
diff
changeset
|
572 |
val _ = Unsynchronized.change skolems (cons (sko_s, ss)) |
11b4395aaf0c
remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
blanchet
parents:
47669
diff
changeset
|
573 |
val sko_t = list_comb (Const (sko_s, rev Ts ---> abs_T), |
11b4395aaf0c
remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
blanchet
parents:
47669
diff
changeset
|
574 |
map Bound (rev js)) |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
575 |
val abs_t = Abs (abs_s, abs_T, |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
576 |
aux ss Ts (incrs js) skolemizable polar t) |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
577 |
in |
47754
11b4395aaf0c
remove too aggressive skolemization optimization (prevented discovery of a model in SYN994^1)
blanchet
parents:
47669
diff
changeset
|
578 |
if null js then |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
579 |
s_betapply Ts (abs_t, sko_t) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
580 |
else |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
581 |
Const (@{const_name Let}, abs_T --> quant_T) $ sko_t |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
582 |
$ abs_t |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
583 |
end |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
584 |
else |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
585 |
raise SAME () |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
586 |
end |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
587 |
else |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
588 |
raise SAME ()) |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
589 |
handle SAME () => |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
590 |
Const (quant_s, quant_T) |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
591 |
$ Abs (abs_s, abs_T, |
38166
28bb89672cc7
fix Skolemizer -- last week's optimizations resulted in UnequalLengths errors
blanchet
parents:
38165
diff
changeset
|
592 |
aux (abs_s :: ss) (abs_T :: Ts) (0 :: incrs js) |
28bb89672cc7
fix Skolemizer -- last week's optimizations resulted in UnequalLengths errors
blanchet
parents:
38165
diff
changeset
|
593 |
(skolemizable andalso |
28bb89672cc7
fix Skolemizer -- last week's optimizations resulted in UnequalLengths errors
blanchet
parents:
38165
diff
changeset
|
594 |
not (is_higher_order_type abs_T)) polar t) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
595 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
596 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
597 |
Const (s0 as @{const_name all}, T0) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
598 |
do_quantifier s0 T0 s1 T1 t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
599 |
| @{const "==>"} $ t1 $ t2 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
600 |
@{const "==>"} $ aux ss Ts js skolemizable (flip_polarity polar) t1 |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
601 |
$ aux ss Ts js skolemizable polar t2 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
602 |
| @{const Pure.conjunction} $ t1 $ t2 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
603 |
@{const Pure.conjunction} $ aux ss Ts js skolemizable polar t1 |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
604 |
$ aux ss Ts js skolemizable polar t2 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
605 |
| @{const Trueprop} $ t1 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
606 |
@{const Trueprop} $ aux ss Ts js skolemizable polar t1 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
607 |
| @{const Not} $ t1 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
608 |
@{const Not} $ aux ss Ts js skolemizable (flip_polarity polar) t1 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
609 |
| Const (s0 as @{const_name All}, T0) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
610 |
do_quantifier s0 T0 s1 T1 t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
611 |
| Const (s0 as @{const_name Ex}, T0) $ Abs (s1, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
612 |
do_quantifier s0 T0 s1 T1 t1 |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
613 |
| @{const HOL.conj} $ t1 $ t2 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
614 |
s_conj (pairself (aux ss Ts js skolemizable polar) (t1, t2)) |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
615 |
| @{const HOL.disj} $ t1 $ t2 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
616 |
s_disj (pairself (aux ss Ts js skolemizable polar) (t1, t2)) |
38786
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
617 |
| @{const HOL.implies} $ t1 $ t2 => |
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
618 |
@{const HOL.implies} $ aux ss Ts js skolemizable (flip_polarity polar) t1 |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
619 |
$ aux ss Ts js skolemizable polar t2 |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
620 |
| (t0 as Const (@{const_name Let}, _)) $ t1 $ t2 => |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
621 |
t0 $ t1 $ aux ss Ts js skolemizable polar t2 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
622 |
| Const (x as (s, T)) => |
38205
37a7272cb453
handle inductive predicates correctly after change in "def" semantics
blanchet
parents:
38204
diff
changeset
|
623 |
if is_real_inductive_pred hol_ctxt x andalso |
37a7272cb453
handle inductive predicates correctly after change in "def" semantics
blanchet
parents:
38204
diff
changeset
|
624 |
not (is_real_equational_fun hol_ctxt x) andalso |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
625 |
not (is_well_founded_inductive_pred hol_ctxt x) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
626 |
let |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
627 |
val gfp = (fixpoint_kind_of_const thy def_tables x = Gfp) |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
628 |
val (pref, connective) = |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
629 |
if gfp then (lbfp_prefix, @{const HOL.disj}) |
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
630 |
else (ubfp_prefix, @{const HOL.conj}) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
631 |
fun pos () = unrolled_inductive_pred_const hol_ctxt gfp x |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
632 |
|> aux ss Ts js skolemizable polar |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
633 |
fun neg () = Const (pref ^ s, T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
634 |
in |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
635 |
case polar |> gfp ? flip_polarity of |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
636 |
Pos => pos () |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
637 |
| Neg => neg () |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
638 |
| Neut => |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
639 |
let |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
640 |
val arg_Ts = binder_types T |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
641 |
fun app f = |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
642 |
list_comb (f (), map Bound (length arg_Ts - 1 downto 0)) |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
643 |
in |
44241 | 644 |
fold_rev absdummy arg_Ts (connective $ app pos $ app neg) |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
645 |
end |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
646 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
647 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
648 |
Const x |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
649 |
| t1 $ t2 => |
38166
28bb89672cc7
fix Skolemizer -- last week's optimizations resulted in UnequalLengths errors
blanchet
parents:
38165
diff
changeset
|
650 |
s_betapply Ts (aux ss Ts js false polar t1, |
28bb89672cc7
fix Skolemizer -- last week's optimizations resulted in UnequalLengths errors
blanchet
parents:
38165
diff
changeset
|
651 |
aux ss Ts js false Neut t2) |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
652 |
| Abs (s, T, t1) => |
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
653 |
Abs (s, T, aux ss Ts (incrs js) skolemizable polar t1) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
654 |
| _ => t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
655 |
end |
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
656 |
in aux [] [] [] true Pos end |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
657 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
658 |
(** Function specialization **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
659 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
660 |
fun params_in_equation (@{const "==>"} $ _ $ t2) = params_in_equation t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
661 |
| params_in_equation (@{const Trueprop} $ t1) = params_in_equation t1 |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
662 |
| params_in_equation (Const (@{const_name HOL.eq}, _) $ t1 $ _) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
663 |
snd (strip_comb t1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
664 |
| params_in_equation _ = [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
665 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
666 |
fun specialize_fun_axiom x x' fixed_js fixed_args extra_args t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
667 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
668 |
val k = fold Integer.max (map maxidx_of_term (fixed_args @ extra_args)) 0 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
669 |
+ 1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
670 |
val t = map_aterms (fn Var ((s, i), T) => Var ((s, k + i), T) | t' => t') t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
671 |
val fixed_params = filter_indices fixed_js (params_in_equation t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
672 |
fun aux args (Abs (s, T, t)) = list_comb (Abs (s, T, aux [] t), args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
673 |
| aux args (t1 $ t2) = aux (aux [] t2 :: args) t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
674 |
| aux args t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
675 |
if t = Const x then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
676 |
list_comb (Const x', extra_args @ filter_out_indices fixed_js args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
677 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
678 |
let val j = find_index (curry (op =) t) fixed_params in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
679 |
list_comb (if j >= 0 then nth fixed_args j else t, args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
680 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
681 |
in aux [] t end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
682 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
683 |
fun static_args_in_term ({ersatz_table, ...} : hol_context) x t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
684 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
685 |
fun fun_calls (Abs (_, _, t)) _ = fun_calls t [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
686 |
| fun_calls (t1 $ t2) args = fun_calls t2 [] #> fun_calls t1 (t2 :: args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
687 |
| fun_calls t args = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
688 |
(case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
689 |
Const (x' as (s', T')) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
690 |
x = x' orelse (case AList.lookup (op =) ersatz_table s' of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
691 |
SOME s'' => x = (s'', T') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
692 |
| NONE => false) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
693 |
| _ => false) ? cons args |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
694 |
fun call_sets [] [] vs = [vs] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
695 |
| call_sets [] uss vs = vs :: call_sets uss [] [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
696 |
| call_sets ([] :: _) _ _ = [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
697 |
| call_sets ((t :: ts) :: tss) uss vs = |
39687 | 698 |
Ord_List.insert Term_Ord.term_ord t vs |> call_sets tss (ts :: uss) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
699 |
val sets = call_sets (fun_calls t [] []) [] [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
700 |
val indexed_sets = sets ~~ (index_seq 0 (length sets)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
701 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
702 |
fold_rev (fn (set, j) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
703 |
case set of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
704 |
[Var _] => AList.lookup (op =) indexed_sets set = SOME j |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
705 |
? cons (j, NONE) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
706 |
| [t as Const _] => cons (j, SOME t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
707 |
| [t as Free _] => cons (j, SOME t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
708 |
| _ => I) indexed_sets [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
709 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
710 |
fun static_args_in_terms hol_ctxt x = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
711 |
map (static_args_in_term hol_ctxt x) |
39687 | 712 |
#> fold1 (Ord_List.inter (prod_ord int_ord (option_ord Term_Ord.term_ord))) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
713 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
714 |
fun overlapping_indices [] _ = [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
715 |
| overlapping_indices _ [] = [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
716 |
| overlapping_indices (ps1 as (j1, t1) :: ps1') (ps2 as (j2, t2) :: ps2') = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
717 |
if j1 < j2 then overlapping_indices ps1' ps2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
718 |
else if j1 > j2 then overlapping_indices ps1 ps2' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
719 |
else overlapping_indices ps1' ps2' |> the_default t2 t1 = t2 ? cons j1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
720 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
721 |
fun special_prefix_for j = special_prefix ^ string_of_int j ^ name_sep |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
722 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
723 |
(* If a constant's definition is picked up deeper than this threshold, we |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
724 |
prevent excessive specialization by not specializing it. *) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
725 |
val special_max_depth = 20 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
726 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
727 |
val bound_var_prefix = "b" |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
728 |
|
38165
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
729 |
fun special_fun_aconv ((x1, js1, ts1), (x2, js2, ts2)) = |
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
730 |
x1 = x2 andalso js1 = js2 andalso length ts1 = length ts2 andalso |
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
731 |
forall (op aconv) (ts1 ~~ ts2) |
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
732 |
|
38204 | 733 |
fun specialize_consts_in_term |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
734 |
(hol_ctxt as {ctxt, thy, stds, specialize, def_tables, simp_table, |
39359 | 735 |
special_funs, ...}) def depth t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
736 |
if not specialize orelse depth > special_max_depth then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
737 |
t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
738 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
739 |
let |
38206 | 740 |
val blacklist = |
741 |
if def then case term_under_def t of Const x => [x] | _ => [] else [] |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
742 |
fun aux args Ts (Const (x as (s, T))) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
743 |
((if not (member (op =) blacklist x) andalso not (null args) andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
744 |
not (String.isPrefix special_prefix s) andalso |
39359 | 745 |
not (is_built_in_const thy stds x) andalso |
38204 | 746 |
(is_equational_fun_but_no_plain_def hol_ctxt x orelse |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
747 |
(is_some (def_of_const thy def_tables x) andalso |
38204 | 748 |
not (is_of_class_const thy x) andalso |
749 |
not (is_constr ctxt stds x) andalso |
|
750 |
not (is_choice_spec_fun hol_ctxt x))) then |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
751 |
let |
41793
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
752 |
val eligible_args = |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
753 |
filter (is_special_eligible_arg true Ts o snd) |
c7a2669ae75d
tweaked Nitpick based on C++ memory model example
blanchet
parents:
41791
diff
changeset
|
754 |
(index_seq 0 (length args) ~~ args) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
755 |
val _ = not (null eligible_args) orelse raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
756 |
val old_axs = equational_fun_axioms hol_ctxt x |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
757 |
|> map (destroy_existential_equalities hol_ctxt) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
758 |
val static_params = static_args_in_terms hol_ctxt x old_axs |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
759 |
val fixed_js = overlapping_indices static_params eligible_args |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
760 |
val _ = not (null fixed_js) orelse raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
761 |
val fixed_args = filter_indices fixed_js args |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
762 |
val vars = fold Term.add_vars fixed_args [] |
35408 | 763 |
|> sort (Term_Ord.fast_indexname_ord o pairself fst) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
764 |
val bound_js = fold (fn t => fn js => add_loose_bnos (t, 0, js)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
765 |
fixed_args [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
766 |
|> sort int_ord |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
767 |
val live_args = filter_out_indices fixed_js args |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
768 |
val extra_args = map Var vars @ map Bound bound_js @ live_args |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
769 |
val extra_Ts = map snd vars @ filter_indices bound_js Ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
770 |
val k = maxidx_of_term t + 1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
771 |
fun var_for_bound_no j = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
772 |
Var ((bound_var_prefix ^ |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
773 |
nat_subscript (find_index (curry (op =) j) bound_js |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
774 |
+ 1), k), |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
775 |
nth Ts j) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
776 |
val fixed_args_in_axiom = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
777 |
map (curry subst_bounds |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
778 |
(map var_for_bound_no (index_seq 0 (length Ts)))) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
779 |
fixed_args |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
780 |
in |
38165
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
781 |
case AList.lookup special_fun_aconv (!special_funs) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
782 |
(x, fixed_js, fixed_args_in_axiom) of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
783 |
SOME x' => list_comb (Const x', extra_args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
784 |
| NONE => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
785 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
786 |
val extra_args_in_axiom = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
787 |
map Var vars @ map var_for_bound_no bound_js |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
788 |
val x' as (s', _) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
789 |
(special_prefix_for (length (!special_funs) + 1) ^ s, |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
790 |
extra_Ts @ filter_out_indices fixed_js (binder_types T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
791 |
---> body_type T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
792 |
val new_axs = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
793 |
map (specialize_fun_axiom x x' fixed_js |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
794 |
fixed_args_in_axiom extra_args_in_axiom) old_axs |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
795 |
val _ = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
796 |
Unsynchronized.change special_funs |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
797 |
(cons ((x, fixed_js, fixed_args_in_axiom), x')) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
798 |
val _ = add_simps simp_table s' new_axs |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
799 |
in list_comb (Const x', extra_args) end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
800 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
801 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
802 |
raise SAME ()) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
803 |
handle SAME () => list_comb (Const x, args)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
804 |
| aux args Ts (Abs (s, T, t)) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
805 |
list_comb (Abs (s, T, aux [] (T :: Ts) t), args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
806 |
| aux args Ts (t1 $ t2) = aux (aux [] Ts t2 :: args) Ts t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
807 |
| aux args _ t = list_comb (t, args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
808 |
in aux [] [] t end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
809 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
810 |
type special_triple = int list * term list * styp |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
811 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
812 |
val cong_var_prefix = "c" |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
813 |
|
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
814 |
fun special_congruence_axiom T (js1, ts1, x1) (js2, ts2, x2) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
815 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
816 |
val (bounds1, bounds2) = pairself (map Var o special_bounds) (ts1, ts2) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
817 |
val Ts = binder_types T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
818 |
val max_j = fold (fold Integer.max) [js1, js2] ~1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
819 |
val (eqs, (args1, args2)) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
820 |
fold (fn j => case pairself (fn ps => AList.lookup (op =) ps j) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
821 |
(js1 ~~ ts1, js2 ~~ ts2) of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
822 |
(SOME t1, SOME t2) => apfst (cons (t1, t2)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
823 |
| (SOME t1, NONE) => apsnd (apsnd (cons t1)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
824 |
| (NONE, SOME t2) => apsnd (apfst (cons t2)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
825 |
| (NONE, NONE) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
826 |
let val v = Var ((cong_var_prefix ^ nat_subscript j, 0), |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
827 |
nth Ts j) in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
828 |
apsnd (pairself (cons v)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
829 |
end) (max_j downto 0) ([], ([], [])) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
830 |
in |
38165
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
831 |
Logic.list_implies (eqs |> filter_out (op aconv) |> distinct (op =) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
832 |
|> map Logic.mk_equals, |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
833 |
Logic.mk_equals (list_comb (Const x1, bounds1 @ args1), |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
834 |
list_comb (Const x2, bounds2 @ args2))) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
835 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
836 |
|
38170 | 837 |
fun special_congruence_axioms (hol_ctxt as {special_funs, ...}) ts = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
838 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
839 |
val groups = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
840 |
!special_funs |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
841 |
|> map (fn ((x, js, ts), x') => (x, (js, ts, x'))) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
842 |
|> AList.group (op =) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
843 |
|> filter_out (is_equational_fun_surely_complete hol_ctxt o fst) |
38170 | 844 |
|> map (fn (x, zs) => |
845 |
(x, zs |> member (op =) ts (Const x) ? cons ([], [], x))) |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
846 |
fun generality (js, _, _) = ~(length js) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
847 |
fun is_more_specific (j1, t1, x1) (j2, t2, x2) = |
38165
9797be44df23
prevent generation of needless specialized constants etc.
blanchet
parents:
37928
diff
changeset
|
848 |
x1 <> x2 andalso length j2 < length j1 andalso |
39687 | 849 |
Ord_List.subset (prod_ord int_ord Term_Ord.term_ord) (j2 ~~ t2, j1 ~~ t1) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
850 |
fun do_pass_1 _ [] [_] [_] = I |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
851 |
| do_pass_1 T skipped _ [] = do_pass_2 T skipped |
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
852 |
| do_pass_1 T skipped all (z :: zs) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
853 |
case filter (is_more_specific z) all |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
854 |
|> sort (int_ord o pairself generality) of |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
855 |
[] => do_pass_1 T (z :: skipped) all zs |
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
856 |
| (z' :: _) => cons (special_congruence_axiom T z z') |
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
857 |
#> do_pass_1 T skipped all zs |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
858 |
and do_pass_2 _ [] = I |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
859 |
| do_pass_2 T (z :: zs) = |
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
860 |
fold (cons o special_congruence_axiom T z) zs #> do_pass_2 T zs |
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
861 |
in fold (fn ((_, T), zs) => do_pass_1 T [] zs zs) groups [] end |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
862 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
863 |
(** Axiom selection **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
864 |
|
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
865 |
fun defined_free_by_assumption t = |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
866 |
let |
47669 | 867 |
fun do_equals u def = |
868 |
if exists_subterm (curry (op aconv) u) def then NONE else SOME u |
|
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
869 |
in |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
870 |
case t of |
47669 | 871 |
Const (@{const_name "=="}, _) $ (u as Free _) $ def => do_equals u def |
872 |
| @{const Trueprop} |
|
873 |
$ (Const (@{const_name HOL.eq}, _) $ (u as Free _) $ def) => |
|
874 |
do_equals u def |
|
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
875 |
| _ => NONE |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
876 |
end |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
877 |
|
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
878 |
fun assumption_exclusively_defines_free assm_ts t = |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
879 |
case defined_free_by_assumption t of |
47669 | 880 |
SOME u => |
881 |
length (filter ((fn SOME u' => u aconv u' | NONE => false) |
|
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
882 |
o defined_free_by_assumption) assm_ts) = 1 |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
883 |
| NONE => false |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
884 |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
885 |
fun all_table_entries table = Symtab.fold (append o snd) table [] |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
886 |
fun extra_table tables s = |
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
887 |
Symtab.make [(s, pairself all_table_entries tables |> op @)] |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
888 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
889 |
fun eval_axiom_for_term j t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
890 |
Logic.mk_equals (Const (eval_prefix ^ string_of_int j, fastype_of t), t) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
891 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
892 |
val is_trivial_equation = the_default false o try (op aconv o Logic.dest_equals) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
893 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
894 |
(* Prevents divergence in case of cyclic or infinite axiom dependencies. *) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
895 |
val axioms_max_depth = 255 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
896 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
897 |
fun axioms_for_term |
35311 | 898 |
(hol_ctxt as {thy, ctxt, max_bisim_depth, stds, user_axioms, |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
899 |
evals, def_tables, nondef_table, choice_spec_table, |
42415
10accf397ab6
use "Spec_Rules" for finding axioms -- more reliable and cleaner
blanchet
parents:
42361
diff
changeset
|
900 |
nondefs, ...}) assm_ts neg_t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
901 |
let |
38170 | 902 |
val (def_assm_ts, nondef_assm_ts) = |
903 |
List.partition (assumption_exclusively_defines_free assm_ts) assm_ts |
|
904 |
val def_assm_table = map (`(the o defined_free_by_assumption)) def_assm_ts |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
905 |
type accumulator = styp list * (term list * term list) |
38206 | 906 |
fun add_axiom get app def depth t (accum as (seen, axs)) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
907 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
908 |
val t = t |> unfold_defs_in_term hol_ctxt |
38206 | 909 |
|> skolemize_term_and_more hol_ctxt ~1 (* FIXME: why ~1? *) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
910 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
911 |
if is_trivial_equation t then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
912 |
accum |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
913 |
else |
38206 | 914 |
let val t' = t |> specialize_consts_in_term hol_ctxt def depth in |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
915 |
if exists (member (op aconv) (get axs)) [t, t'] then accum |
38170 | 916 |
else add_axioms_for_term (depth + 1) t' (seen, app (cons t') axs) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
917 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
918 |
end |
38206 | 919 |
and add_def_axiom depth = add_axiom fst apfst true depth |
920 |
and add_nondef_axiom depth = add_axiom snd apsnd false depth |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
921 |
and add_maybe_def_axiom depth t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
922 |
(if head_of t <> @{const "==>"} then add_def_axiom |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
923 |
else add_nondef_axiom) depth t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
924 |
and add_eq_axiom depth t = |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
925 |
(if is_constr_pattern_formula ctxt t then add_def_axiom |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
926 |
else add_nondef_axiom) depth t |
38170 | 927 |
and add_axioms_for_term depth t (accum as (seen, axs)) = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
928 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
929 |
t1 $ t2 => accum |> fold (add_axioms_for_term depth) [t1, t2] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
930 |
| Const (x as (s, T)) => |
39359 | 931 |
(if member (op aconv) seen t orelse is_built_in_const thy stds x then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
932 |
accum |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
933 |
else |
38170 | 934 |
let val accum = (t :: seen, axs) in |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
935 |
if depth > axioms_max_depth then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
936 |
raise TOO_LARGE ("Nitpick_Preproc.axioms_for_term.\ |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
937 |
\add_axioms_for_term", |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
938 |
"too many nested axioms (" ^ |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
939 |
string_of_int depth ^ ")") |
37260
dde817e6dfb1
added "atoms" option to Nitpick (request from Karlsruhe) + wrap Refute. functions to "nitpick_util.ML"
blanchet
parents:
37256
diff
changeset
|
940 |
else if is_of_class_const thy x then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
941 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
942 |
val class = Logic.class_of_const s |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
943 |
val of_class = Logic.mk_of_class (TVar (("'a", 0), [class]), |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
944 |
class) |
36555
8ff45c2076da
expand combinators in Isar proofs constructed by Sledgehammer;
blanchet
parents:
36389
diff
changeset
|
945 |
val ax1 = try (specialize_type thy x) of_class |
8ff45c2076da
expand combinators in Isar proofs constructed by Sledgehammer;
blanchet
parents:
36389
diff
changeset
|
946 |
val ax2 = Option.map (specialize_type thy x o snd) |
37260
dde817e6dfb1
added "atoms" option to Nitpick (request from Karlsruhe) + wrap Refute. functions to "nitpick_util.ML"
blanchet
parents:
37256
diff
changeset
|
947 |
(get_class_def thy class) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
948 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
949 |
fold (add_maybe_def_axiom depth) (map_filter I [ax1, ax2]) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
950 |
accum |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
951 |
end |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
952 |
else if is_constr ctxt stds x then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
953 |
accum |
37271 | 954 |
else if is_descr (original_name s) then |
955 |
fold (add_nondef_axiom depth) (equational_fun_axioms hol_ctxt x) |
|
956 |
accum |
|
38202
379fb08da97b
prevent the expansion of too large definitions -- use equations for these instead
blanchet
parents:
38190
diff
changeset
|
957 |
else if is_equational_fun_but_no_plain_def hol_ctxt x then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
958 |
fold (add_eq_axiom depth) (equational_fun_axioms hol_ctxt x) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
959 |
accum |
35807
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
blanchet
parents:
35718
diff
changeset
|
960 |
else if is_choice_spec_fun hol_ctxt x then |
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
blanchet
parents:
35718
diff
changeset
|
961 |
fold (add_nondef_axiom depth) |
e4d1b5cbd429
added support for "specification" and "ax_specification" constructs to Nitpick
blanchet
parents:
35718
diff
changeset
|
962 |
(nondef_props_for_const thy true choice_spec_table x) accum |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
963 |
else if is_abs_fun ctxt x then |
38215
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
964 |
accum |> fold (add_nondef_axiom depth) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
965 |
(nondef_props_for_const thy false nondef_table x) |
38240
a44d108a8d39
local versions of Nitpick.register_xxx functions
blanchet
parents:
38215
diff
changeset
|
966 |
|> (is_funky_typedef ctxt (range_type T) orelse |
38215
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
967 |
range_type T = nat_T) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
968 |
? fold (add_maybe_def_axiom depth) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
969 |
(nondef_props_for_const thy true |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
970 |
(extra_table def_tables s) x) |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
971 |
else if is_rep_fun ctxt x then |
38215
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
972 |
accum |> fold (add_nondef_axiom depth) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
973 |
(nondef_props_for_const thy false nondef_table x) |
38240
a44d108a8d39
local versions of Nitpick.register_xxx functions
blanchet
parents:
38215
diff
changeset
|
974 |
|> (is_funky_typedef ctxt (range_type T) orelse |
38215
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
975 |
range_type T = nat_T) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
976 |
? fold (add_maybe_def_axiom depth) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
977 |
(nondef_props_for_const thy true |
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
978 |
(extra_table def_tables s) x) |
38215
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
979 |
|> add_axioms_for_term depth |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
980 |
(Const (mate_of_rep_fun ctxt x)) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
981 |
|> fold (add_def_axiom depth) |
1c7d7eaebdf2
quotient types registered as codatatypes are no longer quotient types
blanchet
parents:
38207
diff
changeset
|
982 |
(inverse_axioms_for_rep_fun ctxt x) |
37253 | 983 |
else if s = @{const_name TYPE} then |
984 |
accum |
|
41791
01d722707a36
always unfold constant defitions marked with "nitpick_def" -- to prevent unfolding, there's already "nitpick_simp"
blanchet
parents:
41052
diff
changeset
|
985 |
else case def_of_const thy def_tables x of |
39345 | 986 |
SOME _ => |
38202
379fb08da97b
prevent the expansion of too large definitions -- use equations for these instead
blanchet
parents:
38190
diff
changeset
|
987 |
fold (add_eq_axiom depth) (equational_fun_axioms hol_ctxt x) |
379fb08da97b
prevent the expansion of too large definitions -- use equations for these instead
blanchet
parents:
38190
diff
changeset
|
988 |
accum |
379fb08da97b
prevent the expansion of too large definitions -- use equations for these instead
blanchet
parents:
38190
diff
changeset
|
989 |
| NONE => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
990 |
accum |> user_axioms <> SOME false |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
991 |
? fold (add_nondef_axiom depth) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
992 |
(nondef_props_for_const thy false nondef_table x) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
993 |
end) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
994 |
|> add_axioms_for_type depth T |
47669 | 995 |
| Free (_, T) => |
38170 | 996 |
(if member (op aconv) seen t then |
997 |
accum |
|
47669 | 998 |
else case AList.lookup (op =) def_assm_table t of |
38170 | 999 |
SOME t => add_def_axiom depth t accum |
1000 |
| NONE => accum) |
|
1001 |
|> add_axioms_for_type depth T |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1002 |
| Var (_, T) => add_axioms_for_type depth T accum |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1003 |
| Bound _ => accum |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1004 |
| Abs (_, T, t) => accum |> add_axioms_for_term depth t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1005 |
|> add_axioms_for_type depth T |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1006 |
and add_axioms_for_type depth T = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1007 |
case T of |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35408
diff
changeset
|
1008 |
Type (@{type_name fun}, Ts) => fold (add_axioms_for_type depth) Ts |
38190
b02e204b613a
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
blanchet
parents:
38170
diff
changeset
|
1009 |
| Type (@{type_name prod}, Ts) => fold (add_axioms_for_type depth) Ts |
46115 | 1010 |
| Type (@{type_name set}, Ts) => fold (add_axioms_for_type depth) Ts |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1011 |
| @{typ prop} => I |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1012 |
| @{typ bool} => I |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1013 |
| TFree (_, S) => add_axioms_for_sort depth T S |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1014 |
| TVar (_, S) => add_axioms_for_sort depth T S |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
1015 |
| Type (z as (_, Ts)) => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1016 |
fold (add_axioms_for_type depth) Ts |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1017 |
#> (if is_pure_typedef ctxt T then |
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1018 |
fold (add_maybe_def_axiom depth) (optimized_typedef_axioms ctxt z) |
38240
a44d108a8d39
local versions of Nitpick.register_xxx functions
blanchet
parents:
38215
diff
changeset
|
1019 |
else if is_quot_type ctxt T then |
35311 | 1020 |
fold (add_def_axiom depth) |
1021 |
(optimized_quot_type_axioms ctxt stds z) |
|
38240
a44d108a8d39
local versions of Nitpick.register_xxx functions
blanchet
parents:
38215
diff
changeset
|
1022 |
else if max_bisim_depth >= 0 andalso is_codatatype ctxt T then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1023 |
fold (add_maybe_def_axiom depth) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1024 |
(codatatype_bisim_axioms hol_ctxt T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1025 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1026 |
I) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1027 |
and add_axioms_for_sort depth T S = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1028 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1029 |
val supers = Sign.complete_sort thy S |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1030 |
val class_axioms = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1031 |
maps (fn class => map prop_of (AxClass.get_info thy class |> #axioms |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1032 |
handle ERROR _ => [])) supers |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1033 |
val monomorphic_class_axioms = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1034 |
map (fn t => case Term.add_tvars t [] of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1035 |
[] => t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1036 |
| [(x, S)] => |
36555
8ff45c2076da
expand combinators in Isar proofs constructed by Sledgehammer;
blanchet
parents:
36389
diff
changeset
|
1037 |
monomorphic_term (Vartab.make [(x, (S, T))]) t |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1038 |
| _ => raise TERM ("Nitpick_Preproc.axioms_for_term.\ |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1039 |
\add_axioms_for_sort", [t])) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1040 |
class_axioms |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1041 |
in fold (add_nondef_axiom depth) monomorphic_class_axioms end |
42415
10accf397ab6
use "Spec_Rules" for finding axioms -- more reliable and cleaner
blanchet
parents:
42361
diff
changeset
|
1042 |
val (mono_nondefs, poly_nondefs) = |
10accf397ab6
use "Spec_Rules" for finding axioms -- more reliable and cleaner
blanchet
parents:
42361
diff
changeset
|
1043 |
List.partition (null o Term.hidden_polymorphism) nondefs |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1044 |
val eval_axioms = map2 eval_axiom_for_term (index_seq 0 (length evals)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1045 |
evals |
38170 | 1046 |
val (seen, (defs, nondefs)) = |
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1047 |
([], ([], [])) |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1048 |
|> add_axioms_for_term 1 neg_t |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1049 |
|> fold_rev (add_nondef_axiom 1) nondef_assm_ts |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1050 |
|> fold_rev (add_def_axiom 1) eval_axioms |
42415
10accf397ab6
use "Spec_Rules" for finding axioms -- more reliable and cleaner
blanchet
parents:
42361
diff
changeset
|
1051 |
|> user_axioms = SOME true ? fold (add_nondef_axiom 1) mono_nondefs |
38170 | 1052 |
val defs = defs @ special_congruence_axioms hol_ctxt seen |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1053 |
val got_all_mono_user_axioms = |
42415
10accf397ab6
use "Spec_Rules" for finding axioms -- more reliable and cleaner
blanchet
parents:
42361
diff
changeset
|
1054 |
(user_axioms = SOME true orelse null mono_nondefs) |
10accf397ab6
use "Spec_Rules" for finding axioms -- more reliable and cleaner
blanchet
parents:
42361
diff
changeset
|
1055 |
in (neg_t :: nondefs, defs, got_all_mono_user_axioms, null poly_nondefs) end |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1056 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1057 |
(** Simplification of constructor/selector terms **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1058 |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1059 |
fun simplify_constrs_and_sels ctxt t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1060 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1061 |
fun is_nth_sel_on t' n (Const (s, _) $ t) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1062 |
(t = t' andalso is_sel_like_and_no_discr s andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1063 |
sel_no_from_name s = n) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1064 |
| is_nth_sel_on _ _ _ = false |
47909
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
1065 |
fun do_term (Const (@{const_name Nitpick.Rep_Frac}, _) |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
1066 |
$ (Const (@{const_name Nitpick.Abs_Frac}, _) $ t1)) [] = |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
1067 |
do_term t1 [] |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
1068 |
| do_term (Const (@{const_name Nitpick.Abs_Frac}, _) |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
1069 |
$ (Const (@{const_name Nitpick.Rep_Frac}, _) $ t1)) [] = |
5f1afeebafbc
fixed "real" after they were redefined as a 'quotient_type'
blanchet
parents:
47754
diff
changeset
|
1070 |
do_term t1 [] |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1071 |
| do_term (t1 $ t2) args = do_term t1 (do_term t2 [] :: args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1072 |
| do_term (t as Const (x as (s, T))) (args as _ :: _) = |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1073 |
((if is_constr_like ctxt x then |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1074 |
if length args = num_binder_types T then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1075 |
case hd args of |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
1076 |
Const (_, T') $ t' => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1077 |
if domain_type T' = body_type T andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1078 |
forall (uncurry (is_nth_sel_on t')) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1079 |
(index_seq 0 (length args) ~~ args) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1080 |
t' |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1081 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1082 |
raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1083 |
| _ => raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1084 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1085 |
raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1086 |
else if is_sel_like_and_no_discr s then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1087 |
case strip_comb (hd args) of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1088 |
(Const (x' as (s', T')), ts') => |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1089 |
if is_constr_like ctxt x' andalso |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1090 |
constr_name_for_sel_like s = s' andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1091 |
not (exists is_pair_type (binder_types T')) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1092 |
list_comb (nth ts' (sel_no_from_name s), tl args) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1093 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1094 |
raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1095 |
| _ => raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1096 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1097 |
raise SAME ()) |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
1098 |
handle SAME () => s_betapplys [] (t, args)) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1099 |
| do_term (Abs (s, T, t')) args = |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
1100 |
s_betapplys [] (Abs (s, T, do_term t' []), args) |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37271
diff
changeset
|
1101 |
| do_term t args = s_betapplys [] (t, args) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1102 |
in do_term t [] end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1103 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1104 |
(** Quantifier massaging: Distributing quantifiers **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1105 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1106 |
fun distribute_quantifiers t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1107 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1108 |
(t0 as Const (@{const_name All}, T0)) $ Abs (s, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1109 |
(case t1 of |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
1110 |
(t10 as @{const HOL.conj}) $ t11 $ t12 => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1111 |
t10 $ distribute_quantifiers (t0 $ Abs (s, T1, t11)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1112 |
$ distribute_quantifiers (t0 $ Abs (s, T1, t12)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1113 |
| (t10 as @{const Not}) $ t11 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1114 |
t10 $ distribute_quantifiers (Const (@{const_name Ex}, T0) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1115 |
$ Abs (s, T1, t11)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1116 |
| t1 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1117 |
if not (loose_bvar1 (t1, 0)) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1118 |
distribute_quantifiers (incr_boundvars ~1 t1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1119 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1120 |
t0 $ Abs (s, T1, distribute_quantifiers t1)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1121 |
| (t0 as Const (@{const_name Ex}, T0)) $ Abs (s, T1, t1) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1122 |
(case distribute_quantifiers t1 of |
38795
848be46708dc
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
haftmann
parents:
38786
diff
changeset
|
1123 |
(t10 as @{const HOL.disj}) $ t11 $ t12 => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1124 |
t10 $ distribute_quantifiers (t0 $ Abs (s, T1, t11)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1125 |
$ distribute_quantifiers (t0 $ Abs (s, T1, t12)) |
38786
e46e7a9cb622
formerly unnamed infix impliciation now named HOL.implies
haftmann
parents:
38240
diff
changeset
|
1126 |
| (t10 as @{const HOL.implies}) $ t11 $ t12 => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1127 |
t10 $ distribute_quantifiers (Const (@{const_name All}, T0) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1128 |
$ Abs (s, T1, t11)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1129 |
$ distribute_quantifiers (t0 $ Abs (s, T1, t12)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1130 |
| (t10 as @{const Not}) $ t11 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1131 |
t10 $ distribute_quantifiers (Const (@{const_name All}, T0) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1132 |
$ Abs (s, T1, t11)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1133 |
| t1 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1134 |
if not (loose_bvar1 (t1, 0)) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1135 |
distribute_quantifiers (incr_boundvars ~1 t1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1136 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1137 |
t0 $ Abs (s, T1, distribute_quantifiers t1)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1138 |
| t1 $ t2 => distribute_quantifiers t1 $ distribute_quantifiers t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1139 |
| Abs (s, T, t') => Abs (s, T, distribute_quantifiers t') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1140 |
| _ => t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1141 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1142 |
(** Quantifier massaging: Pushing quantifiers inward **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1143 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1144 |
fun renumber_bounds j n f t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1145 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1146 |
t1 $ t2 => renumber_bounds j n f t1 $ renumber_bounds j n f t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1147 |
| Abs (s, T, t') => Abs (s, T, renumber_bounds (j + 1) n f t') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1148 |
| Bound j' => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1149 |
Bound (if j' >= j andalso j' < j + n then f (j' - j) + j else j') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1150 |
| _ => t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1151 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1152 |
(* Maximum number of quantifiers in a cluster for which the exponential |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1153 |
algorithm is used. Larger clusters use a heuristic inspired by Claessen & |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1154 |
Soerensson's polynomial binary splitting procedure (p. 5 of their MODEL 2003 |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1155 |
paper). *) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1156 |
val quantifier_cluster_threshold = 7 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1157 |
|
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
1158 |
val push_quantifiers_inward = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1159 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1160 |
fun aux quant_s ss Ts t = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1161 |
(case t of |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
1162 |
Const (s0, _) $ Abs (s1, T1, t1 as _ $ _) => |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1163 |
if s0 = quant_s then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1164 |
aux s0 (s1 :: ss) (T1 :: Ts) t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1165 |
else if quant_s = "" andalso |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1166 |
(s0 = @{const_name All} orelse s0 = @{const_name Ex}) then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1167 |
aux s0 [s1] [T1] t1 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1168 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1169 |
raise SAME () |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1170 |
| _ => raise SAME ()) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1171 |
handle SAME () => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1172 |
case t of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1173 |
t1 $ t2 => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1174 |
if quant_s = "" then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1175 |
aux "" [] [] t1 $ aux "" [] [] t2 |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1176 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1177 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1178 |
fun big_union proj ps = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1179 |
fold (fold (insert (op =)) o proj) ps [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1180 |
val (ts, connective) = strip_any_connective t |
41860
49d0fc8c418c
improved "is_special_eligible_arg" further, by approximating the cardinality of the argument (as is done quite successfully elsewhere)
blanchet
parents:
41803
diff
changeset
|
1181 |
val T_costs = map typical_card_of_type Ts |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1182 |
val t_costs = map size_of_term ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1183 |
val num_Ts = length Ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1184 |
val flip = curry (op -) (num_Ts - 1) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1185 |
val t_boundss = map (map flip o loose_bnos) ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1186 |
fun merge costly_boundss [] = costly_boundss |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1187 |
| merge costly_boundss (j :: js) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1188 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1189 |
val (yeas, nays) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1190 |
List.partition (fn (bounds, _) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1191 |
member (op =) bounds j) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1192 |
costly_boundss |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1193 |
val yeas_bounds = big_union fst yeas |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1194 |
val yeas_cost = Integer.sum (map snd yeas) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1195 |
* nth T_costs j |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1196 |
in merge ((yeas_bounds, yeas_cost) :: nays) js end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1197 |
val cost = Integer.sum o map snd oo merge |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1198 |
fun heuristically_best_permutation _ [] = [] |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1199 |
| heuristically_best_permutation costly_boundss js = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1200 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1201 |
val (costly_boundss, (j, js)) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1202 |
js |> map (`(merge costly_boundss o single)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1203 |
|> sort (int_ord |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1204 |
o pairself (Integer.sum o map snd o fst)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1205 |
|> split_list |>> hd ||> pairf hd tl |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1206 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1207 |
j :: heuristically_best_permutation costly_boundss js |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1208 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1209 |
val js = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1210 |
if length Ts <= quantifier_cluster_threshold then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1211 |
all_permutations (index_seq 0 num_Ts) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1212 |
|> map (`(cost (t_boundss ~~ t_costs))) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1213 |
|> sort (int_ord o pairself fst) |> hd |> snd |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1214 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1215 |
heuristically_best_permutation (t_boundss ~~ t_costs) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1216 |
(index_seq 0 num_Ts) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1217 |
val back_js = map (fn j => find_index (curry (op =) j) js) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1218 |
(index_seq 0 num_Ts) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1219 |
val ts = map (renumber_bounds 0 num_Ts (nth back_js o flip)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1220 |
ts |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1221 |
fun mk_connection [] = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1222 |
raise ARG ("Nitpick_Preproc.push_quantifiers_inward.aux.\ |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1223 |
\mk_connection", "") |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1224 |
| mk_connection ts_cum_bounds = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1225 |
ts_cum_bounds |> map fst |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1226 |
|> foldr1 (fn (t1, t2) => connective $ t1 $ t2) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1227 |
fun build ts_cum_bounds [] = ts_cum_bounds |> mk_connection |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1228 |
| build ts_cum_bounds (j :: js) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1229 |
let |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1230 |
val (yeas, nays) = |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1231 |
List.partition (fn (_, bounds) => |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1232 |
member (op =) bounds j) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1233 |
ts_cum_bounds |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1234 |
||> map (apfst (incr_boundvars ~1)) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1235 |
in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1236 |
if null yeas then |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1237 |
build nays js |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1238 |
else |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1239 |
let val T = nth Ts (flip j) in |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1240 |
build ((Const (quant_s, (T --> bool_T) --> bool_T) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1241 |
$ Abs (nth ss (flip j), T, |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1242 |
mk_connection yeas), |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1243 |
big_union snd yeas) :: nays) js |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1244 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1245 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1246 |
in build (ts ~~ t_boundss) js end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1247 |
| Abs (s, T, t') => Abs (s, T, aux "" [] [] t') |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1248 |
| _ => t |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1249 |
in aux "" [] [] end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1250 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1251 |
(** Preprocessor entry point **) |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1252 |
|
37928
24785fa2416c
do a better job at Skolemizing in Nitpick, for TPTP FOF
blanchet
parents:
37704
diff
changeset
|
1253 |
val max_skolem_depth = 3 |
36389
8228b3a4a2ba
remove "skolemize" option from Nitpick, since Skolemization is always useful
blanchet
parents:
36388
diff
changeset
|
1254 |
|
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1255 |
fun preprocess_formulas |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1256 |
(hol_ctxt as {thy, ctxt, stds, binary_ints, destroy_constrs, boxes, |
41875 | 1257 |
needs, ...}) assm_ts neg_t = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1258 |
let |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1259 |
val (nondef_ts, def_ts, got_all_mono_user_axioms, no_poly_user_axioms) = |
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1260 |
neg_t |> unfold_defs_in_term hol_ctxt |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1261 |
|> close_form |
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1262 |
|> skolemize_term_and_more hol_ctxt max_skolem_depth |
38206 | 1263 |
|> specialize_consts_in_term hol_ctxt false 0 |
38169
b51784515471
optimize local "def"s by treating them as definitions
blanchet
parents:
38166
diff
changeset
|
1264 |
|> axioms_for_term hol_ctxt assm_ts |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1265 |
val binarize = |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
1266 |
is_standard_datatype thy stds nat_T andalso |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1267 |
case binary_ints of |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1268 |
SOME false => false |
35718 | 1269 |
| _ => forall (may_use_binary_ints false) nondef_ts andalso |
1270 |
forall (may_use_binary_ints true) def_ts andalso |
|
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
1271 |
(binary_ints = SOME true orelse |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1272 |
exists should_use_binary_ints (nondef_ts @ def_ts)) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1273 |
val box = exists (not_equal (SOME false) o snd) boxes |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1274 |
val table = |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1275 |
Termtab.empty |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1276 |
|> box ? fold (add_to_uncurry_table ctxt) (nondef_ts @ def_ts) |
41803
ef13e3b7cbaf
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet
parents:
41793
diff
changeset
|
1277 |
fun do_middle def = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1278 |
binarize ? binarize_nat_and_int_in_term |
36388 | 1279 |
#> box ? uncurry_term table |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1280 |
#> box ? box_fun_and_pair_in_term hol_ctxt def |
41803
ef13e3b7cbaf
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet
parents:
41793
diff
changeset
|
1281 |
fun do_tail def = |
46102 | 1282 |
destroy_set_Collect |
1283 |
#> destroy_constrs ? (pull_out_universal_constrs hol_ctxt def |
|
1284 |
#> pull_out_existential_constrs hol_ctxt) |
|
41994
c567c860caf6
always destroy constructor patterns, since this seems to be always useful
blanchet
parents:
41876
diff
changeset
|
1285 |
#> destroy_pulled_out_constrs hol_ctxt def destroy_constrs |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1286 |
#> curry_assms |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1287 |
#> destroy_universal_equalities |
35220
2bcdae5f4fdb
added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s
blanchet
parents:
35190
diff
changeset
|
1288 |
#> destroy_existential_equalities hol_ctxt |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
37253
diff
changeset
|
1289 |
#> simplify_constrs_and_sels ctxt |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1290 |
#> distribute_quantifiers |
35280
54ab4921f826
fixed a few bugs in Nitpick and removed unreferenced variables
blanchet
parents:
35220
diff
changeset
|
1291 |
#> push_quantifiers_inward |
35078
6fd1052fe463
optimization to quantifiers in Nitpick's handling of simp rules + renamed some SAT solvers
blanchet
parents:
35070
diff
changeset
|
1292 |
#> close_form |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1293 |
#> Term.map_abs_vars shortest_name |
41803
ef13e3b7cbaf
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet
parents:
41793
diff
changeset
|
1294 |
val nondef_ts = nondef_ts |> map (do_middle false) |
41875 | 1295 |
val need_ts = |
41876 | 1296 |
case needs of |
1297 |
SOME needs => |
|
1298 |
needs |> map (unfold_defs_in_term hol_ctxt #> do_middle false) |
|
1299 |
| NONE => [] (* FIXME: Implement inference. *) |
|
41803
ef13e3b7cbaf
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet
parents:
41793
diff
changeset
|
1300 |
val nondef_ts = nondef_ts |> map (do_tail false) |
ef13e3b7cbaf
more work on "fix_datatype_vals" optimization (renamed "preconstruct")
blanchet
parents:
41793
diff
changeset
|
1301 |
val def_ts = def_ts |> map (do_middle true #> do_tail true) |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1302 |
in |
41875 | 1303 |
(nondef_ts, def_ts, need_ts, got_all_mono_user_axioms, no_poly_user_axioms, |
1304 |
binarize) |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1305 |
end |
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1306 |
|
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
diff
changeset
|
1307 |
end; |