author | blanchet |
Mon, 06 Dec 2010 13:33:09 +0100 | |
changeset 41002 | 11a442b472c7 |
parent 41001 | 11715564e2ad |
child 41003 | 7e2a7bd55a00 |
permissions | -rw-r--r-- |
33982 | 1 |
(* Title: HOL/Tools/Nitpick/nitpick_mono.ML |
33192 | 2 |
Author: Jasmin Blanchette, TU Muenchen |
34982
7b8c366e34a2
added support for nonstandard models to Nitpick (based on an idea by Koen Claessen) and did other fixes to Nitpick
blanchet
parents:
34936
diff
changeset
|
3 |
Copyright 2009, 2010 |
33192 | 4 |
|
35384 | 5 |
Monotonicity inference for higher-order logic. |
33192 | 6 |
*) |
7 |
||
8 |
signature NITPICK_MONO = |
|
9 |
sig |
|
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
34998
diff
changeset
|
10 |
type hol_context = Nitpick_HOL.hol_context |
33192 | 11 |
|
38179 | 12 |
val trace : bool Unsynchronized.ref |
33192 | 13 |
val formulas_monotonic : |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
14 |
hol_context -> bool -> typ -> term list * term list -> bool |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
15 |
val finitize_funs : |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
16 |
hol_context -> bool -> (typ option * bool option) list -> typ |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
17 |
-> term list * term list -> term list * term list |
33192 | 18 |
end; |
19 |
||
33232
f93390060bbe
internal renaming in Nitpick and fixed Kodkodi invokation on Linux;
blanchet
parents:
33192
diff
changeset
|
20 |
structure Nitpick_Mono : NITPICK_MONO = |
33192 | 21 |
struct |
22 |
||
33232
f93390060bbe
internal renaming in Nitpick and fixed Kodkodi invokation on Linux;
blanchet
parents:
33192
diff
changeset
|
23 |
open Nitpick_Util |
f93390060bbe
internal renaming in Nitpick and fixed Kodkodi invokation on Linux;
blanchet
parents:
33192
diff
changeset
|
24 |
open Nitpick_HOL |
33192 | 25 |
|
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
26 |
structure PL = PropLogic |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
27 |
|
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
28 |
datatype sign = Plus | Minus |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
29 |
|
33192 | 30 |
type var = int |
31 |
||
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
32 |
datatype annotation = Gen | New | Fls | Tru |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
33 |
datatype annotation_atom = A of annotation | V of var |
33192 | 34 |
|
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
35 |
type assign_literal = var * (sign * annotation) |
33192 | 36 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
37 |
datatype mtyp = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
38 |
MAlpha | |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
39 |
MFun of mtyp * annotation_atom * mtyp | |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
40 |
MPair of mtyp * mtyp | |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
41 |
MType of string * mtyp list | |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
42 |
MRec of string * typ list |
33192 | 43 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
44 |
datatype mterm = |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
45 |
MRaw of term * mtyp | |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
46 |
MAbs of string * typ * mtyp * annotation_atom * mterm | |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
47 |
MApp of mterm * mterm |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
48 |
|
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
49 |
type mdata = |
35070
96136eb6218f
split "nitpick_hol.ML" into two files to make it more manageable;
blanchet
parents:
34998
diff
changeset
|
50 |
{hol_ctxt: hol_context, |
35190
ce653cc27a94
make sure that Nitpick uses binary notation consistently if "binary_ints" is enabled
blanchet
parents:
35079
diff
changeset
|
51 |
binarize: bool, |
33192 | 52 |
alpha_T: typ, |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
53 |
no_harmless: bool, |
33192 | 54 |
max_fresh: int Unsynchronized.ref, |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
55 |
datatype_mcache: ((string * typ list) * mtyp) list Unsynchronized.ref, |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
56 |
constr_mcache: (styp * mtyp) list Unsynchronized.ref} |
33192 | 57 |
|
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
58 |
exception UNSOLVABLE of unit |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
59 |
exception MTYPE of string * mtyp list * typ list |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
60 |
exception MTERM of string * mterm list |
33192 | 61 |
|
38179 | 62 |
val trace = Unsynchronized.ref false |
63 |
fun trace_msg msg = if !trace then tracing (msg ()) else () |
|
33192 | 64 |
|
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
65 |
fun string_for_sign Plus = "+" |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
66 |
| string_for_sign Minus = "-" |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
67 |
|
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
68 |
fun negate_sign Plus = Minus |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
69 |
| negate_sign Minus = Plus |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
70 |
|
33192 | 71 |
val string_for_var = signed_string_of_int |
72 |
fun string_for_vars sep [] = "0\<^bsub>" ^ sep ^ "\<^esub>" |
|
73 |
| string_for_vars sep xs = space_implode sep (map string_for_var xs) |
|
74 |
fun subscript_string_for_vars sep xs = |
|
75 |
if null xs then "" else "\<^bsub>" ^ string_for_vars sep xs ^ "\<^esub>" |
|
76 |
||
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
77 |
fun string_for_annotation Gen = "G" |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
78 |
| string_for_annotation New = "N" |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
79 |
| string_for_annotation Fls = "F" |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
80 |
| string_for_annotation Tru = "T" |
33192 | 81 |
|
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
82 |
fun string_for_annotation_atom (A a) = string_for_annotation a |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
83 |
| string_for_annotation_atom (V x) = string_for_var x |
33192 | 84 |
|
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
85 |
fun string_for_assign_literal (x, (sn, a)) = |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
86 |
string_for_var x ^ (case sn of Plus => " = " | Minus => " \<noteq> ") ^ |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
87 |
string_for_annotation a |
33192 | 88 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
89 |
val bool_M = MType (@{type_name bool}, []) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
90 |
val dummy_M = MType (nitpick_prefix ^ "dummy", []) |
33192 | 91 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
92 |
fun is_MRec (MRec _) = true |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
93 |
| is_MRec _ = false |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
94 |
fun dest_MFun (MFun z) = z |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
95 |
| dest_MFun M = raise MTYPE ("Nitpick_Mono.dest_MFun", [M], []) |
33192 | 96 |
|
97 |
val no_prec = 100 |
|
98 |
||
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
99 |
fun precedence_of_mtype (MFun _) = 1 |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
100 |
| precedence_of_mtype (MPair _) = 2 |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
101 |
| precedence_of_mtype _ = no_prec |
33192 | 102 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
103 |
val string_for_mtype = |
33192 | 104 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
105 |
fun aux outer_prec M = |
33192 | 106 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
107 |
val prec = precedence_of_mtype M |
33192 | 108 |
val need_parens = (prec < outer_prec) |
109 |
in |
|
110 |
(if need_parens then "(" else "") ^ |
|
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
111 |
(if M = dummy_M then |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
112 |
"_" |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
113 |
else case M of |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
114 |
MAlpha => "\<alpha>" |
40988 | 115 |
| MFun (M1, aa, M2) => |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
116 |
aux (prec + 1) M1 ^ " \<Rightarrow>\<^bsup>" ^ |
40988 | 117 |
string_for_annotation_atom aa ^ "\<^esup> " ^ aux prec M2 |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
118 |
| MPair (M1, M2) => aux (prec + 1) M1 ^ " \<times> " ^ aux prec M2 |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
119 |
| MType (s, []) => |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
120 |
if s = @{type_name prop} orelse s = @{type_name bool} then "o" |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
121 |
else s |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
122 |
| MType (s, Ms) => "(" ^ commas (map (aux 0) Ms) ^ ") " ^ s |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
123 |
| MRec (s, _) => "[" ^ s ^ "]") ^ |
33192 | 124 |
(if need_parens then ")" else "") |
125 |
end |
|
126 |
in aux 0 end |
|
127 |
||
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
128 |
fun flatten_mtype (MPair (M1, M2)) = maps flatten_mtype [M1, M2] |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
129 |
| flatten_mtype (MType (_, Ms)) = maps flatten_mtype Ms |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
130 |
| flatten_mtype M = [M] |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
131 |
|
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
132 |
fun precedence_of_mterm (MRaw _) = no_prec |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
133 |
| precedence_of_mterm (MAbs _) = 1 |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
134 |
| precedence_of_mterm (MApp _) = 2 |
33192 | 135 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
136 |
fun string_for_mterm ctxt = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
137 |
let |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
138 |
fun mtype_annotation M = "\<^bsup>" ^ string_for_mtype M ^ "\<^esup>" |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
139 |
fun aux outer_prec m = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
140 |
let |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
141 |
val prec = precedence_of_mterm m |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
142 |
val need_parens = (prec < outer_prec) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
143 |
in |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
144 |
(if need_parens then "(" else "") ^ |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
145 |
(case m of |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
146 |
MRaw (t, M) => Syntax.string_of_term ctxt t ^ mtype_annotation M |
40988 | 147 |
| MAbs (s, _, M, aa, m) => |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
148 |
"\<lambda>" ^ s ^ mtype_annotation M ^ ".\<^bsup>" ^ |
40988 | 149 |
string_for_annotation_atom aa ^ "\<^esup> " ^ aux prec m |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
150 |
| MApp (m1, m2) => aux prec m1 ^ " " ^ aux (prec + 1) m2) ^ |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
151 |
(if need_parens then ")" else "") |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
152 |
end |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
153 |
in aux 0 end |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
154 |
|
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
155 |
fun mtype_of_mterm (MRaw (_, M)) = M |
40988 | 156 |
| mtype_of_mterm (MAbs (_, _, M, aa, m)) = MFun (M, aa, mtype_of_mterm m) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
157 |
| mtype_of_mterm (MApp (m1, _)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
158 |
case mtype_of_mterm m1 of |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
159 |
MFun (_, _, M12) => M12 |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
160 |
| M1 => raise MTYPE ("Nitpick_Mono.mtype_of_mterm", [M1], []) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
161 |
|
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
162 |
fun strip_mcomb (MApp (m1, m2)) = strip_mcomb m1 ||> (fn ms => append ms [m2]) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
163 |
| strip_mcomb m = (m, []) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
164 |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
165 |
fun initial_mdata hol_ctxt binarize no_harmless alpha_T = |
35190
ce653cc27a94
make sure that Nitpick uses binary notation consistently if "binary_ints" is enabled
blanchet
parents:
35079
diff
changeset
|
166 |
({hol_ctxt = hol_ctxt, binarize = binarize, alpha_T = alpha_T, |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
167 |
no_harmless = no_harmless, max_fresh = Unsynchronized.ref 0, |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
168 |
datatype_mcache = Unsynchronized.ref [], |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
169 |
constr_mcache = Unsynchronized.ref []} : mdata) |
33192 | 170 |
|
171 |
fun could_exist_alpha_subtype alpha_T (T as Type (_, Ts)) = |
|
34936
c4f04bee79f3
some work on Nitpick's support for quotient types;
blanchet
parents:
34123
diff
changeset
|
172 |
T = alpha_T orelse (not (is_fp_iterator_type T) andalso |
c4f04bee79f3
some work on Nitpick's support for quotient types;
blanchet
parents:
34123
diff
changeset
|
173 |
exists (could_exist_alpha_subtype alpha_T) Ts) |
33192 | 174 |
| could_exist_alpha_subtype alpha_T T = (T = alpha_T) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
175 |
fun could_exist_alpha_sub_mtype _ (alpha_T as TFree _) T = |
34121
5e831d805118
get rid of polymorphic equality in Nitpick's code + a few minor cleanups
blanchet
parents:
33982
diff
changeset
|
176 |
could_exist_alpha_subtype alpha_T T |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
177 |
| could_exist_alpha_sub_mtype ctxt alpha_T T = |
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
178 |
(T = alpha_T orelse is_datatype ctxt [(NONE, true)] T) |
33192 | 179 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
180 |
fun exists_alpha_sub_mtype MAlpha = true |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
181 |
| exists_alpha_sub_mtype (MFun (M1, _, M2)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
182 |
exists exists_alpha_sub_mtype [M1, M2] |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
183 |
| exists_alpha_sub_mtype (MPair (M1, M2)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
184 |
exists exists_alpha_sub_mtype [M1, M2] |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
185 |
| exists_alpha_sub_mtype (MType (_, Ms)) = exists exists_alpha_sub_mtype Ms |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
186 |
| exists_alpha_sub_mtype (MRec _) = true |
33192 | 187 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
188 |
fun exists_alpha_sub_mtype_fresh MAlpha = true |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
189 |
| exists_alpha_sub_mtype_fresh (MFun (_, V _, _)) = true |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
190 |
| exists_alpha_sub_mtype_fresh (MFun (_, _, M2)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
191 |
exists_alpha_sub_mtype_fresh M2 |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
192 |
| exists_alpha_sub_mtype_fresh (MPair (M1, M2)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
193 |
exists exists_alpha_sub_mtype_fresh [M1, M2] |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
194 |
| exists_alpha_sub_mtype_fresh (MType (_, Ms)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
195 |
exists exists_alpha_sub_mtype_fresh Ms |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
196 |
| exists_alpha_sub_mtype_fresh (MRec _) = true |
33192 | 197 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
198 |
fun constr_mtype_for_binders z Ms = |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
199 |
fold_rev (fn M => curry3 MFun M (A Gen)) Ms (MRec z) |
33192 | 200 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
201 |
fun repair_mtype _ _ MAlpha = MAlpha |
40988 | 202 |
| repair_mtype cache seen (MFun (M1, aa, M2)) = |
203 |
MFun (repair_mtype cache seen M1, aa, repair_mtype cache seen M2) |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
204 |
| repair_mtype cache seen (MPair Mp) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
205 |
MPair (pairself (repair_mtype cache seen) Mp) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
206 |
| repair_mtype cache seen (MType (s, Ms)) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
207 |
MType (s, maps (flatten_mtype o repair_mtype cache seen) Ms) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
208 |
| repair_mtype cache seen (MRec (z as (s, _))) = |
33192 | 209 |
case AList.lookup (op =) cache z |> the of |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
210 |
MRec _ => MType (s, []) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
211 |
| M => if member (op =) seen M then MType (s, []) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
212 |
else repair_mtype cache (M :: seen) M |
33192 | 213 |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
214 |
fun repair_datatype_mcache cache = |
33192 | 215 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
216 |
fun repair_one (z, M) = |
33192 | 217 |
Unsynchronized.change cache |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
218 |
(AList.update (op =) (z, repair_mtype (!cache) [] M)) |
33192 | 219 |
in List.app repair_one (rev (!cache)) end |
220 |
||
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
221 |
fun repair_constr_mcache dtype_cache constr_mcache = |
33192 | 222 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
223 |
fun repair_one (x, M) = |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
224 |
Unsynchronized.change constr_mcache |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
225 |
(AList.update (op =) (x, repair_mtype dtype_cache [] M)) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
226 |
in List.app repair_one (!constr_mcache) end |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
227 |
|
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
228 |
fun is_fin_fun_supported_type @{typ prop} = true |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
229 |
| is_fin_fun_supported_type @{typ bool} = true |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
230 |
| is_fin_fun_supported_type (Type (@{type_name option}, _)) = true |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
231 |
| is_fin_fun_supported_type _ = false |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
232 |
fun fin_fun_body _ _ (t as @{term False}) = SOME t |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
233 |
| fin_fun_body _ _ (t as Const (@{const_name None}, _)) = SOME t |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
234 |
| fin_fun_body dom_T ran_T |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
235 |
((t0 as Const (@{const_name If}, _)) |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
236 |
$ (t1 as Const (@{const_name HOL.eq}, _) $ Bound 0 $ t1') |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
237 |
$ t2 $ t3) = |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
238 |
(if loose_bvar1 (t1', 0) then |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
239 |
NONE |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
240 |
else case fin_fun_body dom_T ran_T t3 of |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
241 |
NONE => NONE |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
242 |
| SOME t3 => |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
243 |
SOME (t0 $ (Const (@{const_name is_unknown}, dom_T --> bool_T) $ t1') |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
244 |
$ (Const (@{const_name unknown}, ran_T)) $ (t0 $ t1 $ t2 $ t3))) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
245 |
| fin_fun_body _ _ _ = NONE |
33192 | 246 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
247 |
(* ### FIXME: make sure wellformed! *) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
248 |
|
35672 | 249 |
fun fresh_mfun_for_fun_type (mdata as {max_fresh, ...} : mdata) all_minus |
250 |
T1 T2 = |
|
33192 | 251 |
let |
35672 | 252 |
val M1 = fresh_mtype_for_type mdata all_minus T1 |
253 |
val M2 = fresh_mtype_for_type mdata all_minus T2 |
|
40988 | 254 |
val aa = if not all_minus andalso exists_alpha_sub_mtype_fresh M1 andalso |
255 |
is_fin_fun_supported_type (body_type T2) then |
|
256 |
V (Unsynchronized.inc max_fresh) |
|
257 |
else |
|
258 |
A Gen |
|
259 |
in (M1, aa, M2) end |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
260 |
and fresh_mtype_for_type (mdata as {hol_ctxt as {ctxt, ...}, binarize, alpha_T, |
35672 | 261 |
datatype_mcache, constr_mcache, ...}) |
262 |
all_minus = |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
263 |
let |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
264 |
fun do_type T = |
33192 | 265 |
if T = alpha_T then |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
266 |
MAlpha |
33192 | 267 |
else case T of |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
268 |
Type (@{type_name fun}, [T1, T2]) => |
39342 | 269 |
MFun (fresh_mfun_for_fun_type mdata all_minus T1 T2) |
38190
b02e204b613a
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
blanchet
parents:
38179
diff
changeset
|
270 |
| Type (@{type_name prod}, [T1, T2]) => MPair (pairself do_type (T1, T2)) |
33192 | 271 |
| Type (z as (s, _)) => |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
272 |
if could_exist_alpha_sub_mtype ctxt alpha_T T then |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
273 |
case AList.lookup (op =) (!datatype_mcache) z of |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
274 |
SOME M => M |
33192 | 275 |
| NONE => |
276 |
let |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
277 |
val _ = Unsynchronized.change datatype_mcache (cons (z, MRec z)) |
35219
15a5f213ef5b
fix bug in Nitpick's monotonicity code w.r.t. binary integers
blanchet
parents:
35190
diff
changeset
|
278 |
val xs = binarized_and_boxed_datatype_constrs hol_ctxt binarize T |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
279 |
val (all_Ms, constr_Ms) = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
280 |
fold_rev (fn (_, T') => fn (all_Ms, constr_Ms) => |
33192 | 281 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
282 |
val binder_Ms = map do_type (binder_types T') |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
283 |
val new_Ms = filter exists_alpha_sub_mtype_fresh |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
284 |
binder_Ms |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
285 |
val constr_M = constr_mtype_for_binders z |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
286 |
binder_Ms |
33192 | 287 |
in |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
288 |
(union (op =) new_Ms all_Ms, |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
289 |
constr_M :: constr_Ms) |
33192 | 290 |
end) |
291 |
xs ([], []) |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
292 |
val M = MType (s, all_Ms) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
293 |
val _ = Unsynchronized.change datatype_mcache |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
294 |
(AList.update (op =) (z, M)) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
295 |
val _ = Unsynchronized.change constr_mcache |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
296 |
(append (xs ~~ constr_Ms)) |
33192 | 297 |
in |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
298 |
if forall (not o is_MRec o snd) (!datatype_mcache) then |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
299 |
(repair_datatype_mcache datatype_mcache; |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
300 |
repair_constr_mcache (!datatype_mcache) constr_mcache; |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
301 |
AList.lookup (op =) (!datatype_mcache) z |> the) |
33192 | 302 |
else |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
303 |
M |
33192 | 304 |
end |
305 |
else |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
306 |
MType (s, []) |
37260
dde817e6dfb1
added "atoms" option to Nitpick (request from Karlsruhe) + wrap Refute. functions to "nitpick_util.ML"
blanchet
parents:
37256
diff
changeset
|
307 |
| _ => MType (simple_string_of_typ T, []) |
33192 | 308 |
in do_type end |
309 |
||
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
310 |
fun prodM_factors (MPair (M1, M2)) = maps prodM_factors [M1, M2] |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
311 |
| prodM_factors M = [M] |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
312 |
fun curried_strip_mtype (MFun (M1, _, M2)) = |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
313 |
curried_strip_mtype M2 |>> append (prodM_factors M1) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
314 |
| curried_strip_mtype M = ([], M) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
315 |
fun sel_mtype_from_constr_mtype s M = |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
316 |
let val (arg_Ms, dataM) = curried_strip_mtype M in |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
317 |
MFun (dataM, A Gen, |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
318 |
case sel_no_from_name s of ~1 => bool_M | n => nth arg_Ms n) |
33192 | 319 |
end |
320 |
||
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
321 |
fun mtype_for_constr (mdata as {hol_ctxt = {ctxt, ...}, alpha_T, constr_mcache, |
33192 | 322 |
...}) (x as (_, T)) = |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
323 |
if could_exist_alpha_sub_mtype ctxt alpha_T T then |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
324 |
case AList.lookup (op =) (!constr_mcache) x of |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
325 |
SOME M => M |
35384 | 326 |
| NONE => if T = alpha_T then |
35672 | 327 |
let val M = fresh_mtype_for_type mdata false T in |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
328 |
(Unsynchronized.change constr_mcache (cons (x, M)); M) |
35384 | 329 |
end |
330 |
else |
|
35672 | 331 |
(fresh_mtype_for_type mdata false (body_type T); |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
332 |
AList.lookup (op =) (!constr_mcache) x |> the) |
33192 | 333 |
else |
35672 | 334 |
fresh_mtype_for_type mdata false T |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
335 |
fun mtype_for_sel (mdata as {hol_ctxt, binarize, ...}) (x as (s, _)) = |
35190
ce653cc27a94
make sure that Nitpick uses binary notation consistently if "binary_ints" is enabled
blanchet
parents:
35079
diff
changeset
|
336 |
x |> binarized_and_boxed_constr_for_sel hol_ctxt binarize |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
337 |
|> mtype_for_constr mdata |> sel_mtype_from_constr_mtype s |
33192 | 338 |
|
40989 | 339 |
fun resolve_annotation_atom asgs (V x) = |
340 |
x |> AList.lookup (op =) asgs |> Option.map A |> the_default (V x) |
|
40988 | 341 |
| resolve_annotation_atom _ aa = aa |
40989 | 342 |
fun resolve_mtype asgs = |
33192 | 343 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
344 |
fun aux MAlpha = MAlpha |
40988 | 345 |
| aux (MFun (M1, aa, M2)) = |
40989 | 346 |
MFun (aux M1, resolve_annotation_atom asgs aa, aux M2) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
347 |
| aux (MPair Mp) = MPair (pairself aux Mp) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
348 |
| aux (MType (s, Ms)) = MType (s, map aux Ms) |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
349 |
| aux (MRec z) = MRec z |
33192 | 350 |
in aux end |
351 |
||
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
352 |
datatype comp_op = Eq | Neq | Leq |
33192 | 353 |
|
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
354 |
type comp = annotation_atom * annotation_atom * comp_op * var list |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
355 |
type assign_clause = assign_literal list |
33192 | 356 |
|
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
357 |
type constraint_set = comp list * assign_clause list |
33192 | 358 |
|
359 |
fun string_for_comp_op Eq = "=" |
|
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
360 |
| string_for_comp_op Neq = "\<noteq>" |
33192 | 361 |
| string_for_comp_op Leq = "\<le>" |
362 |
||
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
363 |
fun string_for_comp (aa1, aa2, cmp, xs) = |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
364 |
string_for_annotation_atom aa1 ^ " " ^ string_for_comp_op cmp ^ |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
365 |
subscript_string_for_vars " \<and> " xs ^ " " ^ string_for_annotation_atom aa2 |
33192 | 366 |
|
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
367 |
fun string_for_assign_clause NONE = "\<top>" |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
368 |
| string_for_assign_clause (SOME []) = "\<bot>" |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
369 |
| string_for_assign_clause (SOME asgs) = |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
370 |
space_implode " \<or> " (map string_for_assign_literal asgs) |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
371 |
|
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
372 |
fun add_assign_literal (x, (sn, a)) clauses = |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
373 |
if exists (fn [(x', (sn', a'))] => |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
374 |
x = x' andalso ((sn = sn' andalso a <> a') orelse |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
375 |
(sn <> sn' andalso a = a')) |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
376 |
| _ => false) clauses then |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
377 |
NONE |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
378 |
else |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
379 |
SOME ([(x, a)] :: clauses) |
33192 | 380 |
|
40991
902ad76994d5
proper handling of assignment disjunctions vs. conjunctions
blanchet
parents:
40990
diff
changeset
|
381 |
fun add_assign_disjunct _ NONE = NONE |
902ad76994d5
proper handling of assignment disjunctions vs. conjunctions
blanchet
parents:
40990
diff
changeset
|
382 |
| add_assign_disjunct asg (SOME asgs) = SOME (insert (op =) asg asgs) |
902ad76994d5
proper handling of assignment disjunctions vs. conjunctions
blanchet
parents:
40990
diff
changeset
|
383 |
|
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
384 |
fun add_assign_clause NONE = I |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
385 |
| add_assign_clause (SOME clause) = insert (op =) clause |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
386 |
|
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
387 |
fun annotation_comp Eq a1 a2 = (a1 = a2) |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
388 |
| annotation_comp Neq a1 a2 = (a1 <> a2) |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
389 |
| annotation_comp Leq a1 a2 = (a1 = a2 orelse a2 = Gen) |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
390 |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
391 |
fun sign_for_comp_op Eq = Plus |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
392 |
| sign_for_comp_op Neq = Minus |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
393 |
| sign_for_comp_op Leq = raise BAD ("sign_for_comp_op", "unexpected \"Leq\"") |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
394 |
|
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
395 |
fun do_annotation_atom_comp Leq [] aa1 aa2 (cset as (comps, clauses)) = |
40988 | 396 |
(case (aa1, aa2) of |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
397 |
(A a1, A a2) => if annotation_comp Leq a1 a2 then SOME cset else NONE |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
398 |
| _ => SOME (insert (op =) (aa1, aa2, Leq, []) comps, clauses)) |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
399 |
| do_annotation_atom_comp cmp [] aa1 aa2 (cset as (comps, clauses)) = |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
400 |
(case (aa1, aa2) of |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
401 |
(A a1, A a2) => if annotation_comp cmp a1 a2 then SOME cset else NONE |
40988 | 402 |
| (V x1, A a2) => |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
403 |
clauses |> add_assign_literal (x1, (sign_for_comp_op cmp, a2)) |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
404 |
|> Option.map (pair comps) |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
405 |
| (A _, V _) => do_annotation_atom_comp cmp [] aa2 aa1 cset |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
406 |
| (V _, V _) => SOME (insert (op =) (aa1, aa2, cmp, []) comps, clauses)) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
407 |
| do_annotation_atom_comp cmp xs aa1 aa2 (comps, clauses) = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
408 |
SOME (insert (op =) (aa1, aa2, cmp, xs) comps, clauses) |
33192 | 409 |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
410 |
fun add_annotation_atom_comp cmp xs aa1 aa2 (comps, clauses) = |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
411 |
(trace_msg (fn () => "*** Add " ^ string_for_comp (aa1, aa2, cmp, xs)); |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
412 |
case do_annotation_atom_comp cmp xs aa1 aa2 (comps, clauses) of |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
413 |
NONE => (trace_msg (K "**** Unsolvable"); raise UNSOLVABLE ()) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
414 |
| SOME cset => cset) |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
415 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
416 |
fun do_mtype_comp _ _ _ _ NONE = NONE |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
417 |
| do_mtype_comp _ _ MAlpha MAlpha cset = cset |
40988 | 418 |
| do_mtype_comp Eq xs (MFun (M11, aa1, M12)) (MFun (M21, aa2, M22)) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
419 |
(SOME cset) = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
420 |
cset |> do_annotation_atom_comp Eq xs aa1 aa2 |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
421 |
|> do_mtype_comp Eq xs M11 M21 |> do_mtype_comp Eq xs M12 M22 |
40988 | 422 |
| do_mtype_comp Leq xs (MFun (M11, aa1, M12)) (MFun (M21, aa2, M22)) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
423 |
(SOME cset) = |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
424 |
(if exists_alpha_sub_mtype M11 then |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
425 |
cset |> do_annotation_atom_comp Leq xs aa1 aa2 |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
426 |
|> do_mtype_comp Leq xs M21 M11 |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
427 |
|> (case aa2 of |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
428 |
A Gen => I |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
429 |
| A _ => do_mtype_comp Leq xs M11 M21 |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
430 |
| V x => do_mtype_comp Leq (x :: xs) M11 M21) |
33192 | 431 |
else |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
432 |
SOME cset) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
433 |
|> do_mtype_comp Leq xs M12 M22 |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
434 |
| do_mtype_comp cmp xs (M1 as MPair (M11, M12)) (M2 as MPair (M21, M22)) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
435 |
cset = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
436 |
(cset |> fold (uncurry (do_mtype_comp cmp xs)) [(M11, M21), (M12, M22)] |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
437 |
handle Library.UnequalLengths => |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
438 |
raise MTYPE ("Nitpick_Mono.do_mtype_comp", [M1, M2], [])) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
439 |
| do_mtype_comp _ _ (MType _) (MType _) cset = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
440 |
cset (* no need to compare them thanks to the cache *) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
441 |
| do_mtype_comp cmp _ M1 M2 _ = |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
442 |
raise MTYPE ("Nitpick_Mono.do_mtype_comp (" ^ string_for_comp_op cmp ^ ")", |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
443 |
[M1, M2], []) |
33192 | 444 |
|
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
445 |
fun add_mtype_comp cmp M1 M2 cset = |
40991
902ad76994d5
proper handling of assignment disjunctions vs. conjunctions
blanchet
parents:
40990
diff
changeset
|
446 |
(trace_msg (fn () => "*** Add " ^ string_for_mtype M1 ^ " " ^ |
902ad76994d5
proper handling of assignment disjunctions vs. conjunctions
blanchet
parents:
40990
diff
changeset
|
447 |
string_for_comp_op cmp ^ " " ^ string_for_mtype M2); |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
448 |
case SOME cset |> do_mtype_comp cmp [] M1 M2 of |
40991
902ad76994d5
proper handling of assignment disjunctions vs. conjunctions
blanchet
parents:
40990
diff
changeset
|
449 |
NONE => (trace_msg (K "**** Unsolvable"); raise UNSOLVABLE ()) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
450 |
| SOME cset => cset) |
33192 | 451 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
452 |
val add_mtypes_equal = add_mtype_comp Eq |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
453 |
val add_is_sub_mtype = add_mtype_comp Leq |
33192 | 454 |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
455 |
fun do_notin_mtype_fv _ _ _ NONE = NONE |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
456 |
| do_notin_mtype_fv Minus _ MAlpha cset = cset |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
457 |
| do_notin_mtype_fv Plus [] MAlpha _ = NONE |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
458 |
| do_notin_mtype_fv Plus [asg] MAlpha (SOME clauses) = |
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
459 |
clauses |> add_assign_literal asg |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
460 |
| do_notin_mtype_fv Plus unless MAlpha (SOME clauses) = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
461 |
SOME (insert (op =) unless clauses) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
462 |
| do_notin_mtype_fv sn unless (MFun (M1, A a, M2)) cset = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
463 |
cset |> (if a <> Gen andalso sn = Plus then do_notin_mtype_fv Plus unless M1 |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
464 |
else I) |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
465 |
|> (if a = Gen orelse sn = Plus then do_notin_mtype_fv Minus unless M1 |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
466 |
else I) |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
467 |
|> do_notin_mtype_fv sn unless M2 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
468 |
| do_notin_mtype_fv Plus unless (MFun (M1, V x, M2)) cset = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
469 |
cset |> (case add_assign_disjunct (x, (Plus, Gen)) (SOME unless) of |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
470 |
NONE => I |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
471 |
| SOME unless' => do_notin_mtype_fv Plus unless' M1) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
472 |
|> do_notin_mtype_fv Minus unless M1 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
473 |
|> do_notin_mtype_fv Plus unless M2 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
474 |
| do_notin_mtype_fv Minus unless (MFun (M1, V x, M2)) cset = |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
475 |
cset |> (case fold (fn a => add_assign_disjunct (x, (Plus, a))) [Fls, Tru] |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
476 |
(SOME unless) of |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
477 |
NONE => I |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
478 |
| SOME unless' => do_notin_mtype_fv Plus unless' M1) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
479 |
|> do_notin_mtype_fv Minus unless M2 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
480 |
| do_notin_mtype_fv sn unless (MPair (M1, M2)) cset = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
481 |
cset |> fold (do_notin_mtype_fv sn unless) [M1, M2] |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
482 |
| do_notin_mtype_fv sn unless (MType (_, Ms)) cset = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
483 |
cset |> fold (do_notin_mtype_fv sn unless) Ms |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
484 |
| do_notin_mtype_fv _ _ M _ = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
485 |
raise MTYPE ("Nitpick_Mono.do_notin_mtype_fv", [M], []) |
33192 | 486 |
|
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
487 |
fun add_notin_mtype_fv sn unless M (comps, clauses) = |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
488 |
(trace_msg (fn () => "*** Add " ^ string_for_mtype M ^ " is " ^ |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
489 |
(case sn of Minus => "concrete" | Plus => "complete")); |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
490 |
case SOME clauses |> do_notin_mtype_fv sn unless M of |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
491 |
NONE => (trace_msg (K "**** Unsolvable"); raise UNSOLVABLE ()) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
492 |
| SOME clauses => (comps, clauses)) |
33192 | 493 |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
494 |
val add_mtype_is_concrete = add_notin_mtype_fv Minus |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
495 |
val add_mtype_is_complete = add_notin_mtype_fv Plus |
33192 | 496 |
|
40986
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
497 |
val bool_table = |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
498 |
[(Gen, (false, false)), |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
499 |
(New, (false, true)), |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
500 |
(Fls, (true, false)), |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
501 |
(Tru, (true, true))] |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
502 |
|
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
503 |
fun fst_var n = 2 * n |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
504 |
fun snd_var n = 2 * n + 1 |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
505 |
|
40986
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
506 |
val bools_from_annotation = AList.lookup (op =) bool_table #> the |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
507 |
val annotation_from_bools = AList.find (op =) bool_table #> the_single |
33192 | 508 |
|
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
509 |
fun prop_for_bool b = if b then PL.True else PL.False |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
510 |
fun prop_for_bool_var_equality (v1, v2) = |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
511 |
PL.SAnd (PL.SOr (PL.BoolVar v1, PL.SNot (PL.BoolVar v2)), |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
512 |
PL.SOr (PL.SNot (PL.BoolVar v1), PL.BoolVar v2)) |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
513 |
fun prop_for_assign (x, a) = |
40986
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
514 |
let val (b1, b2) = bools_from_annotation a in |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
515 |
PL.SAnd (PL.BoolVar (fst_var x) |> not b1 ? PL.SNot, |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
516 |
PL.BoolVar (snd_var x) |> not b2 ? PL.SNot) |
40986
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
517 |
end |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
518 |
fun prop_for_assign_literal (x, (Plus, a)) = prop_for_assign (x, a) |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
519 |
| prop_for_assign_literal (x, (Minus, a)) = PL.SNot (prop_for_assign (x, a)) |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
520 |
fun prop_for_atom_assign (A a', a) = prop_for_bool (a = a') |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
521 |
| prop_for_atom_assign (V x, a) = prop_for_assign_literal (x, (Plus, a)) |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
522 |
fun prop_for_atom_equality (aa1, A a2) = prop_for_atom_assign (aa1, a2) |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
523 |
| prop_for_atom_equality (A a1, aa2) = prop_for_atom_assign (aa2, a1) |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
524 |
| prop_for_atom_equality (V x1, V x2) = |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
525 |
PL.SAnd (prop_for_bool_var_equality (pairself fst_var (x1, x2)), |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
526 |
prop_for_bool_var_equality (pairself snd_var (x1, x2))) |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
527 |
val prop_for_assign_clause = PL.exists o map prop_for_assign_literal |
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
528 |
fun prop_for_exists_var_assign_literal xs a = |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
529 |
PL.exists (map (fn x => prop_for_assign_literal (x, (Plus, a))) xs) |
40988 | 530 |
fun prop_for_comp (aa1, aa2, Eq, []) = |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
531 |
PL.SAnd (prop_for_comp (aa1, aa2, Leq, []), |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
532 |
prop_for_comp (aa2, aa1, Leq, [])) |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
533 |
| prop_for_comp (aa1, aa2, Neq, []) = |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
534 |
PL.SNot (prop_for_comp (aa1, aa2, Eq, [])) |
40988 | 535 |
| prop_for_comp (aa1, aa2, Leq, []) = |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
536 |
PL.SOr (prop_for_atom_equality (aa1, aa2), prop_for_atom_assign (aa2, Gen)) |
40988 | 537 |
| prop_for_comp (aa1, aa2, cmp, xs) = |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
538 |
PL.SOr (prop_for_exists_var_assign_literal xs Gen, |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
539 |
prop_for_comp (aa1, aa2, cmp, [])) |
33192 | 540 |
|
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
541 |
fun extract_assigns max_var assigns asgs = |
33192 | 542 |
fold (fn x => fn accum => |
40989 | 543 |
if AList.defined (op =) asgs x then |
33192 | 544 |
accum |
40986
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
545 |
else case (fst_var x, snd_var x) |> pairself assigns of |
cfd91aa80701
use boolean pair to encode annotation, which may now take four values
blanchet
parents:
40985
diff
changeset
|
546 |
(NONE, NONE) => accum |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
547 |
| bp => (x, annotation_from_bools (pairself (the_default false) bp)) |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
548 |
:: accum) |
40989 | 549 |
(max_var downto 1) asgs |
33192 | 550 |
|
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
551 |
fun print_problem comps clauses = |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
552 |
trace_msg (fn () => "*** Problem:\n" ^ |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
553 |
cat_lines (map string_for_comp comps @ |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
554 |
map (string_for_assign_clause o SOME) clauses)) |
33192 | 555 |
|
40989 | 556 |
fun print_solution asgs = |
557 |
trace_msg (fn () => "*** Solution:\n" ^ |
|
558 |
(asgs |
|
559 |
|> map swap |
|
560 |
|> AList.group (op =) |
|
561 |
|> map (fn (a, xs) => string_for_annotation a ^ ": " ^ |
|
562 |
string_for_vars ", " xs) |
|
563 |
|> space_implode "\n")) |
|
33192 | 564 |
|
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
565 |
fun solve max_var (comps, clauses) = |
40146 | 566 |
let |
40996
63112be4a469
added "Neq" operator to monotonicity inference module
blanchet
parents:
40995
diff
changeset
|
567 |
val asgs = map_filter (fn [(x, (_, a))] => SOME (x, a) | _ => NONE) clauses |
40146 | 568 |
fun do_assigns assigns = |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
569 |
SOME (extract_assigns max_var assigns asgs |> tap print_solution) |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
570 |
val _ = print_problem comps clauses |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
571 |
val prop = |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
572 |
PL.all (map prop_for_comp comps @ map prop_for_assign_clause clauses) |
40146 | 573 |
in |
40990
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
574 |
if PL.eval (K false) prop then |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
575 |
do_assigns (K (SOME false)) |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
576 |
else if PL.eval (K true) prop then |
a36d4d869439
adapt monotonicity code to four annotation types
blanchet
parents:
40989
diff
changeset
|
577 |
do_assigns (K (SOME true)) |
40146 | 578 |
else |
579 |
let |
|
580 |
(* use the first ML solver (to avoid startup overhead) *) |
|
581 |
val solvers = !SatSolver.solvers |
|
582 |
|> filter (member (op =) ["dptsat", "dpll"] o fst) |
|
583 |
in |
|
584 |
case snd (hd solvers) prop of |
|
585 |
SatSolver.SATISFIABLE assigns => do_assigns assigns |
|
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
586 |
| _ => (trace_msg (K "*** Unsolvable"); NONE) |
40146 | 587 |
end |
588 |
end |
|
33192 | 589 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
590 |
type mcontext = |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
591 |
{bound_Ts: typ list, |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
592 |
bound_Ms: mtyp list, |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
593 |
frame: (int * annotation_atom) list, |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
594 |
frees: (styp * mtyp) list, |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
595 |
consts: (styp * mtyp) list} |
33192 | 596 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
597 |
fun string_for_bound ctxt Ms (j, aa) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
598 |
Syntax.string_of_term ctxt (Bound (length Ms - j - 1)) ^ " :\<^bsup>" ^ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
599 |
string_for_annotation_atom aa ^ "\<^esup> " ^ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
600 |
string_for_mtype (nth Ms (length Ms - j - 1)) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
601 |
fun string_for_free relevant_frees ((s, _), M) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
602 |
if member (op =) relevant_frees s then SOME (s ^ " : " ^ string_for_mtype M) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
603 |
else NONE |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
604 |
fun string_for_mcontext ctxt t {bound_Ms, frame, frees, ...} = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
605 |
(map_filter (string_for_free (Term.add_free_names t [])) frees @ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
606 |
map (string_for_bound ctxt bound_Ms) frame) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
607 |
|> commas |> enclose "[" "]" |
33192 | 608 |
|
40987
7d52af07bff1
added frame component to Gamma in monotonicity calculus
blanchet
parents:
40986
diff
changeset
|
609 |
val initial_gamma = |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
610 |
{bound_Ts = [], bound_Ms = [], frame = [], frees = [], consts = []} |
33192 | 611 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
612 |
fun push_bound aa T M {bound_Ts, bound_Ms, frame, frees, consts} = |
40987
7d52af07bff1
added frame component to Gamma in monotonicity calculus
blanchet
parents:
40986
diff
changeset
|
613 |
{bound_Ts = T :: bound_Ts, bound_Ms = M :: bound_Ms, |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
614 |
frame = frame @ [(length bound_Ts, aa)], frees = frees, consts = consts} |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
615 |
fun pop_bound {bound_Ts, bound_Ms, frame, frees, consts} = |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
616 |
{bound_Ts = tl bound_Ts, bound_Ms = tl bound_Ms, |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
617 |
frame = frame |> filter_out (fn (j, _) => j = length bound_Ts - 1), |
40987
7d52af07bff1
added frame component to Gamma in monotonicity calculus
blanchet
parents:
40986
diff
changeset
|
618 |
frees = frees, consts = consts} |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
619 |
handle List.Empty => initial_gamma (* FIXME: needed? *) |
33192 | 620 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
621 |
fun set_frame frame ({bound_Ts, bound_Ms, frees, consts, ...} : mcontext) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
622 |
{bound_Ts = bound_Ts, bound_Ms = bound_Ms, frame = frame, frees = frees, |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
623 |
consts = consts} |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
624 |
|
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
625 |
(* FIXME: make sure tracing messages are complete *) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
626 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
627 |
fun add_comp_frame aa cmp = fold (add_annotation_atom_comp cmp [] aa o snd) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
628 |
|
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
629 |
fun add_bound_frame j frame = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
630 |
let |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
631 |
val (new_frame, gen_frame) = List.partition (curry (op =) j o fst) frame |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
632 |
in |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
633 |
add_comp_frame (A New) Leq new_frame |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
634 |
#> add_comp_frame (A Gen) Eq gen_frame |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
635 |
end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
636 |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
637 |
fun fresh_frame ({max_fresh, ...} : mdata) fls tru = |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
638 |
map (apsnd (fn aa => |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
639 |
case (aa, fls, tru) of |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
640 |
(A Fls, SOME a, _) => A a |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
641 |
| (A Tru, _, SOME a) => A a |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
642 |
| (A Gen, _, _) => A Gen |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
643 |
| _ => V (Unsynchronized.inc max_fresh))) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
644 |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
645 |
fun conj_clauses res_aa aa1 aa2 = |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
646 |
[[(aa1, (Neq, Tru)), (aa2, (Neq, Tru)), (res_aa, (Eq, Tru))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
647 |
[(aa1, (Neq, Fls)), (res_aa, (Eq, Fls))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
648 |
[(aa2, (Neq, Fls)), (res_aa, (Eq, Fls))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
649 |
[(aa1, (Neq, Gen)), (aa2, (Eq, Fls)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
650 |
[(aa1, (Neq, New)), (aa2, (Eq, Fls)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
651 |
[(aa1, (Eq, Fls)), (aa2, (Neq, Gen)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
652 |
[(aa1, (Eq, Fls)), (aa2, (Neq, New)), (res_aa, (Eq, Gen))]] |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
653 |
|
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
654 |
fun disj_clauses res_aa aa1 aa2 = |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
655 |
[[(aa1, (Neq, Tru)), (res_aa, (Eq, Tru))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
656 |
[(aa2, (Neq, Tru)), (res_aa, (Eq, Tru))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
657 |
[(aa1, (Neq, Fls)), (aa2, (Neq, Fls)), (res_aa, (Eq, Fls))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
658 |
[(aa1, (Neq, Gen)), (aa2, (Eq, Tru)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
659 |
[(aa1, (Neq, New)), (aa2, (Eq, Tru)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
660 |
[(aa1, (Eq, Tru)), (aa2, (Neq, Gen)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
661 |
[(aa1, (Eq, Tru)), (aa2, (Neq, New)), (res_aa, (Eq, Gen))]] |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
662 |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
663 |
fun imp_clauses res_aa aa1 aa2 = |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
664 |
[[(aa1, (Neq, Fls)), (res_aa, (Eq, Tru))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
665 |
[(aa2, (Neq, Tru)), (res_aa, (Eq, Tru))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
666 |
[(aa1, (Neq, Tru)), (aa2, (Neq, Fls)), (res_aa, (Eq, Fls))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
667 |
[(aa1, (Neq, Gen)), (aa2, (Eq, Tru)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
668 |
[(aa1, (Neq, New)), (aa2, (Eq, Tru)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
669 |
[(aa1, (Eq, Fls)), (aa2, (Neq, Gen)), (res_aa, (Eq, Gen))], |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
670 |
[(aa1, (Eq, Fls)), (aa2, (Neq, New)), (res_aa, (Eq, Gen))]] |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
671 |
|
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
672 |
fun add_annotation_clause_from_quasi_clause _ NONE = NONE |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
673 |
| add_annotation_clause_from_quasi_clause [] accum = accum |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
674 |
| add_annotation_clause_from_quasi_clause ((aa, (cmp, a)) :: rest) accum = |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
675 |
case aa of |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
676 |
A a' => if annotation_comp cmp a' a then NONE |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
677 |
else add_annotation_clause_from_quasi_clause rest accum |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
678 |
| V x => add_annotation_clause_from_quasi_clause rest accum |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
679 |
|> Option.map (cons (x, (sign_for_comp_op cmp, a))) |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
680 |
|
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
681 |
fun assign_clause_from_quasi_clause unless = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
682 |
add_annotation_clause_from_quasi_clause unless (SOME []) |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
683 |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
684 |
fun add_connective_var conn mk_quasi_clauses res_aa aa1 aa2 = |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
685 |
(trace_msg (fn () => "*** Add " ^ string_for_annotation_atom res_aa ^ " = " ^ |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
686 |
string_for_annotation_atom aa1 ^ " " ^ conn ^ " " ^ |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
687 |
string_for_annotation_atom aa2); |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
688 |
fold (add_assign_clause o assign_clause_from_quasi_clause) |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
689 |
(mk_quasi_clauses res_aa aa1 aa2)) |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
690 |
fun add_connective_frames conn mk_quasi_clauses res_frame frame1 frame2 = |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
691 |
fold I (map3 (fn (_, res_aa) => fn (_, aa1) => fn (_, aa2) => |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
692 |
add_connective_var conn mk_quasi_clauses res_aa aa1 aa2) |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
693 |
res_frame frame1 frame2) |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
694 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
695 |
fun kill_unused_in_frame is_in (accum as ({frame, ...}, _)) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
696 |
let val (used_frame, unused_frame) = List.partition is_in frame in |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
697 |
accum |>> set_frame used_frame |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
698 |
||> add_comp_frame (A Gen) Eq unused_frame |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
699 |
end |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
700 |
|
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
701 |
fun split_frame is_in_fun (gamma as {frame, ...}, cset) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
702 |
let |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
703 |
fun bubble fun_frame arg_frame [] cset = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
704 |
((rev fun_frame, rev arg_frame), cset) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
705 |
| bubble fun_frame arg_frame ((bound as (_, aa)) :: rest) cset = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
706 |
if is_in_fun bound then |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
707 |
bubble (bound :: fun_frame) arg_frame rest |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
708 |
(cset |> add_comp_frame aa Leq arg_frame) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
709 |
else |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
710 |
bubble fun_frame (bound :: arg_frame) rest cset |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
711 |
in cset |> bubble [] [] frame ||> pair gamma end |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
712 |
|
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
713 |
fun add_annotation_atom_comp_alt _ (A Gen) _ _ = I |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
714 |
| add_annotation_atom_comp_alt _ (A _) _ _ = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
715 |
(trace_msg (K "*** Expected G"); raise UNSOLVABLE ()) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
716 |
| add_annotation_atom_comp_alt cmp (V x) aa1 aa2 = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
717 |
add_annotation_atom_comp cmp [x] aa1 aa2 |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
718 |
|
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
719 |
fun add_arg_order1 ((_, aa), (_, prev_aa)) = I |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
720 |
add_annotation_atom_comp_alt Neq prev_aa (A Gen) aa |
40999
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
721 |
fun add_app1 fun_aa ((_, res_aa), (_, arg_aa)) = I |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
722 |
let |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
723 |
val clause = [(arg_aa, (Eq, New)), (res_aa, (Eq, Gen))] |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
724 |
|> assign_clause_from_quasi_clause |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
725 |
in |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
726 |
trace_msg (fn () => "*** Add " ^ string_for_assign_clause clause); |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
727 |
apsnd (add_assign_clause clause) |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
728 |
#> add_annotation_atom_comp_alt Leq arg_aa fun_aa res_aa |
69d0d445c46a
fixed bug in clause handling in monotonicity code, whereby the unsound rule False | x <--> False was used to simplify constraints
blanchet
parents:
40998
diff
changeset
|
729 |
end |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
730 |
fun add_app _ [] [] = I |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
731 |
| add_app fun_aa res_frame arg_frame = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
732 |
add_comp_frame (A New) Leq arg_frame |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
733 |
#> fold add_arg_order1 (tl arg_frame ~~ (fst (split_last arg_frame))) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
734 |
#> fold (add_app1 fun_aa) (res_frame ~~ arg_frame) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
735 |
|
39359 | 736 |
fun consider_term (mdata as {hol_ctxt = {thy, ctxt, stds, ...}, alpha_T, |
737 |
max_fresh, ...}) = |
|
33192 | 738 |
let |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
739 |
fun is_enough_eta_expanded t = |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
740 |
case strip_comb t of |
39359 | 741 |
(Const x, ts) => the_default 0 (arity_of_built_in_const thy stds x) |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
742 |
<= length ts |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
743 |
| _ => true |
35672 | 744 |
val mtype_for = fresh_mtype_for_type mdata false |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
745 |
fun plus_set_mtype_for_dom M = |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
746 |
MFun (M, A (if exists_alpha_sub_mtype M then Fls else Gen), bool_M) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
747 |
fun do_all T (gamma, cset) = |
33192 | 748 |
let |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
749 |
val abs_M = mtype_for (domain_type (domain_type T)) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
750 |
val body_M = mtype_for (body_type T) |
33192 | 751 |
in |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
752 |
(MFun (MFun (abs_M, A Gen, body_M), A Gen, body_M), |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
753 |
(gamma, cset |> add_mtype_is_complete [] abs_M)) |
33192 | 754 |
end |
755 |
fun do_equals T (gamma, cset) = |
|
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
756 |
let |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
757 |
val M = mtype_for (domain_type T) |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
758 |
val aa = V (Unsynchronized.inc max_fresh) |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
759 |
in |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
760 |
(MFun (M, A Gen, MFun (M, aa, mtype_for (nth_range_type 2 T))), |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
761 |
(gamma, cset |> add_mtype_is_concrete [] M |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
762 |
|> add_annotation_atom_comp Leq [] (A Fls) aa)) |
33192 | 763 |
end |
764 |
fun do_robust_set_operation T (gamma, cset) = |
|
765 |
let |
|
766 |
val set_T = domain_type T |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
767 |
val M1 = mtype_for set_T |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
768 |
val M2 = mtype_for set_T |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
769 |
val M3 = mtype_for set_T |
33192 | 770 |
in |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
771 |
(MFun (M1, A Gen, MFun (M2, A Gen, M3)), |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
772 |
(gamma, cset |> add_is_sub_mtype M1 M3 |> add_is_sub_mtype M2 M3)) |
33192 | 773 |
end |
774 |
fun do_fragile_set_operation T (gamma, cset) = |
|
775 |
let |
|
776 |
val set_T = domain_type T |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
777 |
val set_M = mtype_for set_T |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
778 |
fun custom_mtype_for (T as Type (@{type_name fun}, [T1, T2])) = |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
779 |
if T = set_T then set_M |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
780 |
else MFun (custom_mtype_for T1, A Gen, custom_mtype_for T2) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
781 |
| custom_mtype_for T = mtype_for T |
33192 | 782 |
in |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
783 |
(custom_mtype_for T, (gamma, cset |> add_mtype_is_concrete [] set_M)) |
33192 | 784 |
end |
785 |
fun do_pair_constr T accum = |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
786 |
case mtype_for (nth_range_type 2 T) of |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
787 |
M as MPair (a_M, b_M) => |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
788 |
(MFun (a_M, A Gen, MFun (b_M, A Gen, M)), accum) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
789 |
| M => raise MTYPE ("Nitpick_Mono.consider_term.do_pair_constr", [M], []) |
33192 | 790 |
fun do_nth_pair_sel n T = |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
791 |
case mtype_for (domain_type T) of |
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
792 |
M as MPair (a_M, b_M) => |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
793 |
pair (MFun (M, A Gen, if n = 0 then a_M else b_M)) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
794 |
| M => raise MTYPE ("Nitpick_Mono.consider_term.do_nth_pair_sel", [M], []) |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
795 |
and do_connect conn mk_quasi_clauses t0 t1 t2 (accum as ({frame, ...}, _)) = |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
796 |
let |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
797 |
val frame1 = fresh_frame mdata (SOME Tru) NONE frame |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
798 |
val frame2 = fresh_frame mdata (SOME Fls) NONE frame |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
799 |
val (m1, accum) = accum |>> set_frame frame1 |> do_term t1 |
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
800 |
val (m2, accum) = accum |>> set_frame frame2 |> do_term t2 |
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
801 |
in |
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
802 |
(MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2), |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
803 |
accum |>> set_frame frame |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
804 |
||> apsnd (add_connective_frames conn mk_quasi_clauses |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
805 |
frame frame1 frame2)) |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
806 |
end |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
807 |
and do_term t |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
808 |
(accum as (gamma as {bound_Ts, bound_Ms, frame, frees, consts}, |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
809 |
cset)) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
810 |
(trace_msg (fn () => " " ^ string_for_mcontext ctxt t gamma ^ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
811 |
" \<turnstile> " ^ Syntax.string_of_term ctxt t ^ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
812 |
" : _?"); |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
813 |
case t of |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
814 |
@{const False} => |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
815 |
(MRaw (t, bool_M), accum ||> add_comp_frame (A Fls) Leq frame) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
816 |
| @{const True} => |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
817 |
(MRaw (t, bool_M), accum ||> add_comp_frame (A Tru) Leq frame) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
818 |
| Const (x as (s, T)) => |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
819 |
(case AList.lookup (op =) consts x of |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
820 |
SOME M => (M, accum) |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
821 |
| NONE => |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
822 |
if not (could_exist_alpha_subtype alpha_T T) then |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
823 |
(mtype_for T, accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
824 |
else case s of |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
825 |
@{const_name all} => do_all T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
826 |
| @{const_name "=="} => do_equals T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
827 |
| @{const_name All} => do_all T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
828 |
| @{const_name Ex} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
829 |
let val set_T = domain_type T in |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
830 |
do_term (Abs (Name.uu, set_T, |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
831 |
@{const Not} $ (HOLogic.mk_eq |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
832 |
(Abs (Name.uu, domain_type set_T, |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
833 |
@{const False}), |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
834 |
Bound 0)))) accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
835 |
|>> mtype_of_mterm |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
836 |
end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
837 |
| @{const_name HOL.eq} => do_equals T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
838 |
| @{const_name The} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
839 |
(trace_msg (K "*** The"); raise UNSOLVABLE ()) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
840 |
| @{const_name Eps} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
841 |
(trace_msg (K "*** Eps"); raise UNSOLVABLE ()) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
842 |
| @{const_name If} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
843 |
do_robust_set_operation (range_type T) accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
844 |
|>> curry3 MFun bool_M (A Gen) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
845 |
| @{const_name Pair} => do_pair_constr T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
846 |
| @{const_name fst} => do_nth_pair_sel 0 T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
847 |
| @{const_name snd} => do_nth_pair_sel 1 T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
848 |
| @{const_name Id} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
849 |
(MFun (mtype_for (domain_type T), A Gen, bool_M), accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
850 |
| @{const_name converse} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
851 |
let |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
852 |
val x = Unsynchronized.inc max_fresh |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
853 |
fun mtype_for_set T = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
854 |
MFun (mtype_for (domain_type T), V x, bool_M) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
855 |
val ab_set_M = domain_type T |> mtype_for_set |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
856 |
val ba_set_M = range_type T |> mtype_for_set |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
857 |
in (MFun (ab_set_M, A Gen, ba_set_M), accum) end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
858 |
| @{const_name trancl} => do_fragile_set_operation T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
859 |
| @{const_name rel_comp} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
860 |
let |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
861 |
val x = Unsynchronized.inc max_fresh |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
862 |
fun mtype_for_set T = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
863 |
MFun (mtype_for (domain_type T), V x, bool_M) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
864 |
val bc_set_M = domain_type T |> mtype_for_set |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
865 |
val ab_set_M = domain_type (range_type T) |> mtype_for_set |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
866 |
val ac_set_M = nth_range_type 2 T |> mtype_for_set |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
867 |
in |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
868 |
(MFun (bc_set_M, A Gen, MFun (ab_set_M, A Gen, ac_set_M)), |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
869 |
accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
870 |
end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
871 |
| @{const_name image} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
872 |
let |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
873 |
val a_M = mtype_for (domain_type (domain_type T)) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
874 |
val b_M = mtype_for (range_type (domain_type T)) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
875 |
in |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
876 |
(MFun (MFun (a_M, A Gen, b_M), A Gen, |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
877 |
MFun (plus_set_mtype_for_dom a_M, A Gen, |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
878 |
plus_set_mtype_for_dom b_M)), accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
879 |
end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
880 |
| @{const_name finite} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
881 |
let val M1 = mtype_for (domain_type (domain_type T)) in |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
882 |
(MFun (plus_set_mtype_for_dom M1, A Gen, bool_M), accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
883 |
end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
884 |
| @{const_name Sigma} => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
885 |
let |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
886 |
val x = Unsynchronized.inc max_fresh |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
887 |
fun mtype_for_set T = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
888 |
MFun (mtype_for (domain_type T), V x, bool_M) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
889 |
val a_set_T = domain_type T |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
890 |
val a_M = mtype_for (domain_type a_set_T) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
891 |
val b_set_M = |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
892 |
mtype_for_set (range_type (domain_type (range_type T))) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
893 |
val a_set_M = mtype_for_set a_set_T |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
894 |
val a_to_b_set_M = MFun (a_M, A Gen, b_set_M) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
895 |
val ab_set_M = mtype_for_set (nth_range_type 2 T) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
896 |
in |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
897 |
(MFun (a_set_M, A Gen, MFun (a_to_b_set_M, A Gen, ab_set_M)), |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
898 |
accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
899 |
end |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
900 |
| _ => |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
901 |
if s = @{const_name safe_The} then |
33192 | 902 |
let |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
903 |
val a_set_M = mtype_for (domain_type T) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
904 |
val a_M = dest_MFun a_set_M |> #1 |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
905 |
in (MFun (a_set_M, A Gen, a_M), accum) end |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
906 |
else if s = @{const_name ord_class.less_eq} andalso |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
907 |
is_set_type (domain_type T) then |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
908 |
do_fragile_set_operation T accum |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
909 |
else if is_sel s then |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
910 |
(mtype_for_sel mdata x, accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
911 |
else if is_constr ctxt stds x then |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
912 |
(mtype_for_constr mdata x, accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
913 |
else if is_built_in_const thy stds x then |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
914 |
(fresh_mtype_for_type mdata true T, accum) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
915 |
else |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
916 |
let val M = mtype_for T in |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
917 |
(M, ({bound_Ts = bound_Ts, bound_Ms = bound_Ms, frame = frame, |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
918 |
frees = frees, consts = (x, M) :: consts}, cset)) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
919 |
end) |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
920 |
|>> curry MRaw t |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
921 |
||> apsnd (add_comp_frame (A Gen) Eq frame) |
33192 | 922 |
| Free (x as (_, T)) => |
923 |
(case AList.lookup (op =) frees x of |
|
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
924 |
SOME M => (M, accum) |
33192 | 925 |
| NONE => |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
926 |
let val M = mtype_for T in |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
927 |
(M, ({bound_Ts = bound_Ts, bound_Ms = bound_Ms, frame = frame, |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
928 |
frees = (x, M) :: frees, consts = consts}, cset)) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
929 |
end) |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
930 |
|>> curry MRaw t ||> apsnd (add_comp_frame (A Gen) Eq frame) |
38179 | 931 |
| Var _ => (trace_msg (K "*** Var"); raise UNSOLVABLE ()) |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
932 |
| Bound j => |
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
933 |
(MRaw (t, nth bound_Ms j), |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
934 |
accum ||> add_bound_frame (length bound_Ts - j - 1) frame) |
35385
29f81babefd7
improved precision of infinite "shallow" datatypes in Nitpick;
blanchet
parents:
35384
diff
changeset
|
935 |
| Abs (s, T, t') => |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
936 |
(case fin_fun_body T (fastype_of1 (T :: bound_Ts, t')) t' of |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
937 |
SOME t' => |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
938 |
let |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
939 |
val M = mtype_for T |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
940 |
val (m', accum) = do_term t' (accum |>> push_bound (A Fls) T M) |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
941 |
in (MAbs (s, T, M, A Fls, m'), accum |>> pop_bound) end |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
942 |
| NONE => |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
943 |
((case t' of |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
944 |
t1' $ Bound 0 => |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
945 |
if not (loose_bvar1 (t1', 0)) andalso |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
946 |
is_enough_eta_expanded t1' then |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
947 |
do_term (incr_boundvars ~1 t1') accum |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
948 |
else |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
949 |
raise SAME () |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
950 |
| (t11 as Const (@{const_name HOL.eq}, _)) $ Bound 0 $ t13 => |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
951 |
if not (loose_bvar1 (t13, 0)) then |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
952 |
do_term (incr_boundvars ~1 (t11 $ t13)) accum |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
953 |
else |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
954 |
raise SAME () |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
955 |
| _ => raise SAME ()) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
956 |
handle SAME () => |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
957 |
let |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
958 |
val M = mtype_for T |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
959 |
val aa = V (Unsynchronized.inc max_fresh) |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
960 |
val (m', accum) = |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
961 |
do_term t' (accum |>> push_bound aa T M) |
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
962 |
in (MAbs (s, T, M, aa, m'), accum |>> pop_bound) end)) |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
963 |
| @{const Not} $ t1 => |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
964 |
do_connect "\<implies>" imp_clauses @{const implies} t1 |
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
965 |
@{const False} accum |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
966 |
| (t0 as @{const conj}) $ t1 $ t2 => |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
967 |
do_connect "\<and>" conj_clauses t0 t1 t2 accum |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
968 |
| (t0 as @{const disj}) $ t1 $ t2 => |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
969 |
do_connect "\<or>" disj_clauses t0 t1 t2 accum |
40995
3cae30b60577
started implementing connectives in new monotonicity calculus
blanchet
parents:
40994
diff
changeset
|
970 |
| (t0 as @{const implies}) $ t1 $ t2 => |
40997
67e11a73532a
implemented connectives in new monotonicity calculus
blanchet
parents:
40996
diff
changeset
|
971 |
do_connect "\<implies>" imp_clauses t0 t1 t2 accum |
33192 | 972 |
| Const (@{const_name Let}, _) $ t1 $ t2 => |
973 |
do_term (betapply (t2, t1)) accum |
|
974 |
| t1 $ t2 => |
|
975 |
let |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
976 |
fun is_in t (j, _) = loose_bvar1 (t, length bound_Ts - j - 1) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
977 |
val accum as ({frame, ...}, _) = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
978 |
accum |> kill_unused_in_frame (is_in t) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
979 |
val ((frame1a, frame1b), accum) = accum |> split_frame (is_in t1) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
980 |
val frame2a = frame1a |> map (apsnd (K (A Gen))) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
981 |
val frame2b = |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
982 |
frame1b |> map (apsnd (fn _ => V (Unsynchronized.inc max_fresh))) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
983 |
val frame2 = frame2a @ frame2b |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
984 |
val (m1, accum) = accum |>> set_frame frame1a |> do_term t1 |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
985 |
val (m2, accum) = accum |>> set_frame frame2 |> do_term t2 |
33192 | 986 |
in |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
987 |
let |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
988 |
val (M11, aa, _) = mtype_of_mterm m1 |> dest_MFun |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
989 |
val M2 = mtype_of_mterm m2 |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
990 |
in |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
991 |
(MApp (m1, m2), |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
992 |
accum |>> set_frame frame |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
993 |
||> add_is_sub_mtype M2 M11 |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
994 |
||> add_app aa frame1b frame2b) |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
995 |
end |
33192 | 996 |
end) |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
997 |
|> tap (fn (m, (gamma, _)) => |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
998 |
trace_msg (fn () => " " ^ string_for_mcontext ctxt t gamma ^ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
999 |
" \<turnstile> " ^ |
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
1000 |
string_for_mterm ctxt m)) |
33192 | 1001 |
in do_term end |
1002 |
||
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1003 |
fun force_gen_funs 0 _ = I |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1004 |
| force_gen_funs n (M as MFun (M1, _, M2)) = |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1005 |
add_mtypes_equal M (MFun (M1, A Gen, M2)) #> force_gen_funs (n - 1) M2 |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1006 |
| force_gen_funs _ M = raise MTYPE ("Nitpick_Mono.force_gen_funs", [M], []) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1007 |
fun consider_general_equals mdata def (x as (_, T)) t1 t2 accum = |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1008 |
let |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1009 |
val (m1, accum) = consider_term mdata t1 accum |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1010 |
val (m2, accum) = consider_term mdata t2 accum |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1011 |
val M1 = mtype_of_mterm m1 |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1012 |
val M2 = mtype_of_mterm m2 |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1013 |
val accum = accum ||> add_mtypes_equal M1 M2 |
35672 | 1014 |
val body_M = fresh_mtype_for_type mdata false (nth_range_type 2 T) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1015 |
val m = MApp (MApp (MRaw (Const x, |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1016 |
MFun (M1, A Gen, MFun (M2, A Fls, body_M))), m1), m2) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1017 |
in |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1018 |
(m, if def then |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1019 |
let val (head_m, arg_ms) = strip_mcomb m1 in |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1020 |
accum ||> force_gen_funs (length arg_ms) (mtype_of_mterm head_m) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1021 |
end |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1022 |
else |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1023 |
accum) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1024 |
end |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1025 |
|
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1026 |
fun consider_general_formula (mdata as {hol_ctxt = {ctxt, ...}, max_fresh, |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1027 |
...}) = |
33192 | 1028 |
let |
35672 | 1029 |
val mtype_for = fresh_mtype_for_type mdata false |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1030 |
val do_term = consider_term mdata |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
1031 |
fun do_formula sn t (accum as (gamma, _)) = |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1032 |
let |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1033 |
fun do_quantifier (quant_x as (quant_s, _)) abs_s abs_T body_t = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1034 |
let |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1035 |
val abs_M = mtype_for abs_T |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1036 |
val x = Unsynchronized.inc max_fresh |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1037 |
val side_cond = ((sn = Minus) = (quant_s = @{const_name Ex})) |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1038 |
fun ann () = if quant_s = @{const_name Ex} then Fls else Tru |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1039 |
val (body_m, accum) = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1040 |
accum ||> side_cond |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1041 |
? add_mtype_is_complete [(x, (Minus, ann ()))] abs_M |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1042 |
|>> push_bound (V x) abs_T abs_M |> do_formula sn body_t |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1043 |
val body_M = mtype_of_mterm body_m |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1044 |
in |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1045 |
(MApp (MRaw (Const quant_x, |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1046 |
MFun (MFun (abs_M, A Gen, body_M), A Gen, body_M)), |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1047 |
MAbs (abs_s, abs_T, abs_M, A Gen, body_m)), |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1048 |
accum |>> pop_bound) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1049 |
end |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1050 |
fun do_equals x t1 t2 = |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1051 |
case sn of |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1052 |
Plus => do_term t accum |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1053 |
| Minus => consider_general_equals mdata false x t1 t2 accum |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1054 |
in |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1055 |
(trace_msg (fn () => " " ^ string_for_mcontext ctxt t gamma ^ |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1056 |
" \<turnstile> " ^ Syntax.string_of_term ctxt t ^ |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1057 |
" : o\<^sup>" ^ string_for_sign sn ^ "?"); |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1058 |
case t of |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1059 |
Const (x as (@{const_name all}, _)) $ Abs (s1, T1, t1) => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1060 |
do_quantifier x s1 T1 t1 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1061 |
| Const (x as (@{const_name "=="}, _)) $ t1 $ t2 => do_equals x t1 t2 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1062 |
| @{const Trueprop} $ t1 => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1063 |
let val (m1, accum) = do_formula sn t1 accum in |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1064 |
(MApp (MRaw (@{const Trueprop}, mtype_for (bool_T --> prop_T)), |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1065 |
m1), accum) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1066 |
end |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1067 |
| @{const Not} $ t1 => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1068 |
let val (m1, accum) = do_formula (negate_sign sn) t1 accum in |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1069 |
(MApp (MRaw (@{const Not}, mtype_for (bool_T --> bool_T)), m1), |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1070 |
accum) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1071 |
end |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1072 |
| Const (x as (@{const_name All}, _)) $ Abs (s1, T1, t1) => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1073 |
do_quantifier x s1 T1 t1 |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1074 |
| Const (x0 as (@{const_name Ex}, T0)) $ (t1 as Abs (s1, T1, t1')) => |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1075 |
(case sn of |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1076 |
Plus => do_quantifier x0 s1 T1 t1' |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1077 |
| Minus => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1078 |
(* FIXME: Move elsewhere *) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1079 |
do_term (@{const Not} |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1080 |
$ (HOLogic.eq_const (domain_type T0) $ t1 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1081 |
$ Abs (Name.uu, T1, @{const False}))) accum) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1082 |
| Const (x as (@{const_name HOL.eq}, _)) $ t1 $ t2 => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1083 |
do_equals x t1 t2 |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1084 |
| Const (@{const_name Let}, _) $ t1 $ t2 => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1085 |
do_formula sn (betapply (t2, t1)) accum |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1086 |
| (t0 as Const (s0, _)) $ t1 $ t2 => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1087 |
if s0 = @{const_name "==>"} orelse |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1088 |
s0 = @{const_name Pure.conjunction} orelse |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1089 |
s0 = @{const_name conj} orelse s0 = @{const_name disj} orelse |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1090 |
s0 = @{const_name implies} then |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1091 |
let |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1092 |
val impl = (s0 = @{const_name "==>"} orelse |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1093 |
s0 = @{const_name implies}) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1094 |
val (m1, accum) = do_formula (sn |> impl ? negate_sign) t1 accum |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1095 |
val (m2, accum) = do_formula sn t2 accum |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1096 |
in |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1097 |
(MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2), |
37704
c6161bee8486
adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
blanchet
parents:
37678
diff
changeset
|
1098 |
accum) |
c6161bee8486
adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
blanchet
parents:
37678
diff
changeset
|
1099 |
end |
41000
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1100 |
else |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1101 |
do_term t accum |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1102 |
| _ => do_term t accum) |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1103 |
end |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1104 |
|> tap (fn (m, (gamma, _)) => |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1105 |
trace_msg (fn () => string_for_mcontext ctxt t gamma ^ |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1106 |
" \<turnstile> " ^ |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1107 |
string_for_mterm ctxt m ^ " : o\<^sup>" ^ |
4bbff1684465
implemented All rules from new monotonicity calculus
blanchet
parents:
40999
diff
changeset
|
1108 |
string_for_sign sn)) |
33192 | 1109 |
in do_formula end |
1110 |
||
1111 |
(* The harmless axiom optimization below is somewhat too aggressive in the face |
|
1112 |
of (rather peculiar) user-defined axioms. *) |
|
1113 |
val harmless_consts = |
|
1114 |
[@{const_name ord_class.less}, @{const_name ord_class.less_eq}] |
|
1115 |
val bounteous_consts = [@{const_name bisim}] |
|
1116 |
||
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1117 |
fun is_harmless_axiom ({no_harmless = true, ...} : mdata) _ = false |
39359 | 1118 |
| is_harmless_axiom {hol_ctxt = {thy, stds, ...}, ...} t = |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1119 |
Term.add_consts t [] |
39359 | 1120 |
|> filter_out (is_built_in_const thy stds) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1121 |
|> (forall (member (op =) harmless_consts o original_name o fst) orf |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1122 |
exists (member (op =) bounteous_consts o fst)) |
33192 | 1123 |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1124 |
fun consider_nondefinitional_axiom mdata t = |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1125 |
if is_harmless_axiom mdata t then pair (MRaw (t, dummy_M)) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1126 |
else consider_general_formula mdata Plus t |
33192 | 1127 |
|
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
1128 |
fun consider_definitional_axiom (mdata as {hol_ctxt = {ctxt, ...}, ...}) t = |
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
1129 |
if not (is_constr_pattern_formula ctxt t) then |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1130 |
consider_nondefinitional_axiom mdata t |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1131 |
else if is_harmless_axiom mdata t then |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1132 |
pair (MRaw (t, dummy_M)) |
33192 | 1133 |
else |
1134 |
let |
|
35672 | 1135 |
val mtype_for = fresh_mtype_for_type mdata false |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1136 |
val do_term = consider_term mdata |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1137 |
fun do_all quant_t abs_s abs_T body_t accum = |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1138 |
let |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1139 |
val abs_M = mtype_for abs_T |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1140 |
val (body_m, accum) = |
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
1141 |
accum |>> push_bound (A Gen) abs_T abs_M |> do_formula body_t |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1142 |
val body_M = mtype_of_mterm body_m |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1143 |
in |
40985
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
1144 |
(MApp (MRaw (quant_t, MFun (MFun (abs_M, A Gen, body_M), A Gen, |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
1145 |
body_M)), |
8b870370c26f
started generalizing monotonicity code to accommodate new calculus
blanchet
parents:
40722
diff
changeset
|
1146 |
MAbs (abs_s, abs_T, abs_M, A Gen, body_m)), |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1147 |
accum |>> pop_bound) |
33192 | 1148 |
end |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1149 |
and do_conjunction t0 t1 t2 accum = |
33192 | 1150 |
let |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1151 |
val (m1, accum) = do_formula t1 accum |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1152 |
val (m2, accum) = do_formula t2 accum |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1153 |
in |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1154 |
(MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2), accum) |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1155 |
end |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1156 |
and do_implies t0 t1 t2 accum = |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1157 |
let |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1158 |
val (m1, accum) = do_term t1 accum |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1159 |
val (m2, accum) = do_formula t2 accum |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1160 |
in |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1161 |
(MApp (MApp (MRaw (t0, mtype_for (fastype_of t0)), m1), m2), accum) |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1162 |
end |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1163 |
and do_formula t accum = |
41002 | 1164 |
case t of |
1165 |
(t0 as Const (@{const_name all}, _)) $ Abs (s1, T1, t1) => |
|
1166 |
do_all t0 s1 T1 t1 accum |
|
1167 |
| @{const Trueprop} $ t1 => |
|
1168 |
let val (m1, accum) = do_formula t1 accum in |
|
1169 |
(MApp (MRaw (@{const Trueprop}, mtype_for (bool_T --> prop_T)), m1), |
|
1170 |
accum) |
|
1171 |
end |
|
1172 |
| Const (x as (@{const_name "=="}, _)) $ t1 $ t2 => |
|
1173 |
consider_general_equals mdata true x t1 t2 accum |
|
1174 |
| (t0 as @{const "==>"}) $ t1 $ t2 => do_implies t0 t1 t2 accum |
|
1175 |
| (t0 as @{const Pure.conjunction}) $ t1 $ t2 => |
|
1176 |
do_conjunction t0 t1 t2 accum |
|
1177 |
| (t0 as Const (@{const_name All}, _)) $ Abs (s0, T1, t1) => |
|
1178 |
do_all t0 s0 T1 t1 accum |
|
1179 |
| Const (x as (@{const_name HOL.eq}, _)) $ t1 $ t2 => |
|
1180 |
consider_general_equals mdata true x t1 t2 accum |
|
1181 |
| (t0 as @{const conj}) $ t1 $ t2 => do_conjunction t0 t1 t2 accum |
|
1182 |
| (t0 as @{const implies}) $ t1 $ t2 => do_implies t0 t1 t2 accum |
|
1183 |
| _ => raise TERM ("Nitpick_Mono.consider_definitional_axiom.\ |
|
1184 |
\do_formula", [t]) |
|
33192 | 1185 |
in do_formula t end |
1186 |
||
40989 | 1187 |
fun string_for_mtype_of_term ctxt asgs t M = |
1188 |
Syntax.string_of_term ctxt t ^ " : " ^ string_for_mtype (resolve_mtype asgs M) |
|
33192 | 1189 |
|
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
1190 |
fun print_mcontext ctxt asgs ({frees, consts, ...} : mcontext) = |
38179 | 1191 |
trace_msg (fn () => |
40989 | 1192 |
map (fn (x, M) => string_for_mtype_of_term ctxt asgs (Free x) M) frees @ |
1193 |
map (fn (x, M) => string_for_mtype_of_term ctxt asgs (Const x) M) consts |
|
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1194 |
|> cat_lines) |
33192 | 1195 |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1196 |
fun amass f t (ms, accum) = |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1197 |
let val (m, accum) = f t accum in (m :: ms, accum) end |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1198 |
|
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1199 |
fun infer which no_harmless (hol_ctxt as {ctxt, ...}) binarize alpha_T |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1200 |
(nondef_ts, def_ts) = |
33192 | 1201 |
let |
38179 | 1202 |
val _ = trace_msg (fn () => "****** " ^ which ^ " analysis: " ^ |
1203 |
string_for_mtype MAlpha ^ " is " ^ |
|
1204 |
Syntax.string_of_typ ctxt alpha_T) |
|
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1205 |
val mdata as {max_fresh, constr_mcache, ...} = |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1206 |
initial_mdata hol_ctxt binarize no_harmless alpha_T |
40994
3bdb8df0daf0
more work on frames in the new monotonicity calculus
blanchet
parents:
40993
diff
changeset
|
1207 |
val accum = (initial_gamma, ([], [])) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1208 |
val (nondef_ms, accum) = |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1209 |
([], accum) |> amass (consider_general_formula mdata Plus) (hd nondef_ts) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1210 |
|> fold (amass (consider_nondefinitional_axiom mdata)) |
35386
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1211 |
(tl nondef_ts) |
45a4e19d3ebd
more work on the new monotonicity stuff in Nitpick
blanchet
parents:
35385
diff
changeset
|
1212 |
val (def_ms, (gamma, cset)) = |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1213 |
([], accum) |> fold (amass (consider_definitional_axiom mdata)) def_ts |
33192 | 1214 |
in |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1215 |
case solve (!max_fresh) cset of |
40998
bcd23ddeecef
started implementing the new monotonicity rules for application
blanchet
parents:
40997
diff
changeset
|
1216 |
SOME asgs => (print_mcontext ctxt asgs gamma; |
40989 | 1217 |
SOME (asgs, (nondef_ms, def_ms), !constr_mcache)) |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1218 |
| _ => NONE |
33192 | 1219 |
end |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1220 |
handle UNSOLVABLE () => NONE |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1221 |
| MTYPE (loc, Ms, Ts) => |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1222 |
raise BAD (loc, commas (map string_for_mtype Ms @ |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1223 |
map (Syntax.string_of_typ ctxt) Ts)) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1224 |
| MTERM (loc, ms) => |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1225 |
raise BAD (loc, commas (map (string_for_mterm ctxt) ms)) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1226 |
|
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1227 |
val formulas_monotonic = is_some oooo infer "Monotonicity" false |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1228 |
|
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1229 |
fun fin_fun_constr T1 T2 = |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1230 |
(@{const_name FinFun}, (T1 --> T2) --> Type (@{type_name fin_fun}, [T1, T2])) |
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1231 |
|
40993
52ee2a187cdb
support 3 monotonicity calculi in one and fix soundness bug
blanchet
parents:
40991
diff
changeset
|
1232 |
fun finitize_funs (hol_ctxt as {thy, ctxt, stds, constr_cache, ...}) binarize |
41001
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1233 |
finitizes alpha_T tsp = |
11715564e2ad
removed old baggage from monotonicity calculus -- the "calculus" option didn't really work anyway because of on-the-fly simplifications
blanchet
parents:
41000
diff
changeset
|
1234 |
case infer "Finiteness" true hol_ctxt binarize alpha_T tsp of |
40989 | 1235 |
SOME (asgs, msp, constr_mtypes) => |
1236 |
if forall (curry (op =) Gen o snd) asgs then |
|
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1237 |
tsp |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1238 |
else |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1239 |
let |
40988 | 1240 |
fun should_finitize T aa = |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1241 |
case triple_lookup (type_match thy) finitizes T of |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1242 |
SOME (SOME false) => false |
40989 | 1243 |
| _ => resolve_annotation_atom asgs aa = A Fls |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1244 |
fun type_from_mtype T M = |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1245 |
case (M, T) of |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1246 |
(MAlpha, _) => T |
40988 | 1247 |
| (MFun (M1, aa, M2), Type (@{type_name fun}, Ts)) => |
1248 |
Type (if should_finitize T aa then @{type_name fin_fun} |
|
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1249 |
else @{type_name fun}, map2 type_from_mtype Ts [M1, M2]) |
38190
b02e204b613a
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
blanchet
parents:
38179
diff
changeset
|
1250 |
| (MPair (M1, M2), Type (@{type_name prod}, Ts)) => |
b02e204b613a
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
blanchet
parents:
38179
diff
changeset
|
1251 |
Type (@{type_name prod}, map2 type_from_mtype Ts [M1, M2]) |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1252 |
| (MType _, _) => T |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1253 |
| _ => raise MTYPE ("Nitpick_Mono.finitize_funs.type_from_mtype", |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1254 |
[M], [T]) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1255 |
fun finitize_constr (x as (s, T)) = |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1256 |
(s, case AList.lookup (op =) constr_mtypes x of |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1257 |
SOME M => type_from_mtype T M |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1258 |
| NONE => T) |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1259 |
fun term_from_mterm new_Ts old_Ts m = |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1260 |
case m of |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1261 |
MRaw (t, M) => |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1262 |
let |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1263 |
val T = fastype_of1 (old_Ts, t) |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1264 |
val T' = type_from_mtype T M |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1265 |
in |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1266 |
case t of |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1267 |
Const (x as (s, _)) => |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1268 |
if s = @{const_name finite} then |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1269 |
case domain_type T' of |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1270 |
set_T' as Type (@{type_name fin_fun}, _) => |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1271 |
Abs (Name.uu, set_T', @{const True}) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1272 |
| _ => Const (s, T') |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1273 |
else if s = @{const_name "=="} orelse |
38864
4abe644fcea5
formerly unnamed infix equality now named HOL.eq
haftmann
parents:
38795
diff
changeset
|
1274 |
s = @{const_name HOL.eq} then |
37476
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1275 |
let |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1276 |
val T = |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1277 |
case T' of |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1278 |
Type (_, [T1, Type (_, [T2, T3])]) => |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1279 |
T1 --> T2 --> T3 |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1280 |
| _ => raise TYPE ("Nitpick_Mono.finitize_funs.\ |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1281 |
\term_from_mterm", [T, T'], []) |
0681e46b4022
optimized code generated for datatype cases + more;
blanchet
parents:
37267
diff
changeset
|
1282 |
in coerce_term hol_ctxt new_Ts T' T (Const (s, T)) end |
39359 | 1283 |
else if is_built_in_const thy stds x then |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1284 |
coerce_term hol_ctxt new_Ts T' T t |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
1285 |
else if is_constr ctxt stds x then |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1286 |
Const (finitize_constr x) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1287 |
else if is_sel s then |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1288 |
let |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1289 |
val n = sel_no_from_name s |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1290 |
val x' = |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1291 |
x |> binarized_and_boxed_constr_for_sel hol_ctxt binarize |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1292 |
|> finitize_constr |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1293 |
val x'' = |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1294 |
binarized_and_boxed_nth_sel_for_constr hol_ctxt binarize |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1295 |
x' n |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1296 |
in Const x'' end |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1297 |
else |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1298 |
Const (s, T') |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1299 |
| Free (s, T) => Free (s, type_from_mtype T M) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1300 |
| Bound _ => t |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1301 |
| _ => raise MTERM ("Nitpick_Mono.finitize_funs.term_from_mterm", |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1302 |
[m]) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1303 |
end |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1304 |
| MApp (m1, m2) => |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1305 |
let |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1306 |
val (t1, t2) = pairself (term_from_mterm new_Ts old_Ts) (m1, m2) |
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1307 |
val (T1, T2) = pairself (curry fastype_of1 new_Ts) (t1, t2) |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1308 |
val (t1', T2') = |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1309 |
case T1 of |
39316
b6c4385ab400
change defaults of Auto Nitpick so that it consumes less resources (time and Kodkod threads)
blanchet
parents:
38864
diff
changeset
|
1310 |
Type (s, [T11, T12]) => |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1311 |
(if s = @{type_name fin_fun} then |
37256
0dca1ec52999
thread along context instead of theory for typedef lookup
blanchet
parents:
36385
diff
changeset
|
1312 |
select_nth_constr_arg ctxt stds (fin_fun_constr T11 T12) t1 |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1313 |
0 (T11 --> T12) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1314 |
else |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1315 |
t1, T11) |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1316 |
| _ => raise TYPE ("Nitpick_Mono.finitize_funs.term_from_mterm", |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1317 |
[T1], []) |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1318 |
in betapply (t1', coerce_term hol_ctxt new_Ts T2' T2 t2) end |
40988 | 1319 |
| MAbs (s, old_T, M, aa, m') => |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1320 |
let |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1321 |
val new_T = type_from_mtype old_T M |
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1322 |
val t' = term_from_mterm (new_T :: new_Ts) (old_T :: old_Ts) m' |
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1323 |
val T' = fastype_of1 (new_T :: new_Ts, t') |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1324 |
in |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1325 |
Abs (s, new_T, t') |
40988 | 1326 |
|> should_finitize (new_T --> T') aa |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1327 |
? construct_value ctxt stds (fin_fun_constr new_T T') o single |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1328 |
end |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1329 |
in |
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1330 |
Unsynchronized.change constr_cache (map (apsnd (map finitize_constr))); |
37267
5c47d633c84d
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
blanchet
parents:
37260
diff
changeset
|
1331 |
pairself (map (term_from_mterm [] [])) msp |
35812
394fe2b064cd
solve error in "Nitpick_Mono" + short path when no finite functions are inferred
blanchet
parents:
35672
diff
changeset
|
1332 |
end |
35665
ff2bf50505ab
added "finitize" option to Nitpick + remove dependency on "Coinductive_List"
blanchet
parents:
35386
diff
changeset
|
1333 |
| NONE => tsp |
33192 | 1334 |
|
1335 |
end; |