author | ballarin |
Tue, 16 Sep 2008 12:27:05 +0200 | |
changeset 28236 | c447b60d67f5 |
parent 28110 | 9d121b171a0a |
child 28259 | 5b2af04ec9fb |
permissions | -rw-r--r-- |
12014 | 1 |
(* Title: Pure/Isar/locale.ML |
11896 | 2 |
ID: $Id$ |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
3 |
Author: Clemens Ballarin, TU Muenchen; Markus Wenzel, LMU/TU Muenchen |
11896 | 4 |
|
12058 | 5 |
Locales -- Isar proof contexts as meta-level predicates, with local |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
6 |
syntax and implicit structures. |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
7 |
|
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
8 |
Draws basic ideas from Florian Kammueller's original version of |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
9 |
locales, but uses the richer infrastructure of Isar instead of the raw |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
10 |
meta-logic. Furthermore, structured import of contexts (with merge |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
11 |
and rename operations) are provided, as well as type-inference of the |
13375 | 12 |
signature parts, and predicate definitions of the specification text. |
14446 | 13 |
|
17437 | 14 |
Interpretation enables the reuse of theorems of locales in other |
15 |
contexts, namely those defined by theories, structured proofs and |
|
16 |
locales themselves. |
|
17 |
||
14446 | 18 |
See also: |
19 |
||
20 |
[1] Clemens Ballarin. Locales and Locale Expressions in Isabelle/Isar. |
|
21 |
In Stefano Berardi et al., Types for Proofs and Programs: International |
|
15099 | 22 |
Workshop, TYPES 2003, Torino, Italy, LNCS 3085, pages 34-50, 2004. |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
23 |
[2] Clemens Ballarin. Interpretation of Locales in Isabelle: Managing |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
24 |
Dependencies between Locales. Technical Report TUM-I0607, Technische |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
25 |
Universitaet Muenchen, 2006. |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
26 |
[3] Clemens Ballarin. Interpretation of Locales in Isabelle: Theories and |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
27 |
Proof Contexts. In J.M. Borwein and W.M. Farmer, MKM 2006, LNAI 4108, |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
28 |
pages 31-43, 2006. |
11896 | 29 |
*) |
30 |
||
16169
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
31 |
(* TODO: |
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
32 |
- beta-eta normalisation of interpretation parameters |
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
33 |
- dangling type frees in locales |
16620
2a7f46324218
Proper treatment of beta-redexes in witness theorems.
ballarin
parents:
16458
diff
changeset
|
34 |
- test subsumption of interpretations when merging theories |
16169
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
35 |
*) |
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
36 |
|
11896 | 37 |
signature LOCALE = |
38 |
sig |
|
12273 | 39 |
datatype expr = |
40 |
Locale of string | |
|
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
41 |
Rename of expr * (string * mixfix option) option list | |
12273 | 42 |
Merge of expr list |
43 |
val empty: expr |
|
18137 | 44 |
datatype 'a element = Elem of 'a | Expr of expr |
21035 | 45 |
val map_elem: ('a -> 'b) -> 'a element -> 'b element |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
46 |
|
16458 | 47 |
val intern: theory -> xstring -> string |
24751 | 48 |
val intern_expr: theory -> expr -> expr |
16458 | 49 |
val extern: theory -> string -> xstring |
19991
0c9650664d47
Locales no longer generate views. The following functions have changed
ballarin
parents:
19984
diff
changeset
|
50 |
val init: string -> theory -> Proof.context |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
51 |
|
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
52 |
(* The specification of a locale *) |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
53 |
val parameters_of: theory -> string -> ((string * typ) * mixfix) list |
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
54 |
val parameters_of_expr: theory -> expr -> ((string * typ) * mixfix) list |
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
55 |
val local_asms_of: theory -> string -> (Attrib.binding * term list) list |
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
56 |
val global_asms_of: theory -> string -> (Attrib.binding * term list) list |
27716 | 57 |
|
58 |
(* Theorems *) |
|
25619 | 59 |
val intros: theory -> string -> thm list * thm list |
60 |
val dests: theory -> string -> thm list |
|
27716 | 61 |
(* Not part of the official interface. DO NOT USE *) |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
62 |
val facts_of: theory -> string -> (Attrib.binding * (thm list * Attrib.src list) list) list list |
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
63 |
|
18899
a8e913c93578
theorem(_in_locale): Element.statement, Obtain.statement;
wenzelm
parents:
18890
diff
changeset
|
64 |
(* Processing of locale statements *) |
18137 | 65 |
val read_context_statement: xstring option -> Element.context element list -> |
19585 | 66 |
(string * string list) list list -> Proof.context -> |
19991
0c9650664d47
Locales no longer generate views. The following functions have changed
ballarin
parents:
19984
diff
changeset
|
67 |
string option * Proof.context * Proof.context * (term * term list) list list |
21035 | 68 |
val read_context_statement_i: string option -> Element.context element list -> |
69 |
(string * string list) list list -> Proof.context -> |
|
70 |
string option * Proof.context * Proof.context * (term * term list) list list |
|
18137 | 71 |
val cert_context_statement: string option -> Element.context_i element list -> |
19585 | 72 |
(term * term list) list list -> Proof.context -> |
19991
0c9650664d47
Locales no longer generate views. The following functions have changed
ballarin
parents:
19984
diff
changeset
|
73 |
string option * Proof.context * Proof.context * (term * term list) list list |
19780 | 74 |
val read_expr: expr -> Element.context list -> Proof.context -> |
75 |
Element.context_i list * Proof.context |
|
76 |
val cert_expr: expr -> Element.context_i list -> Proof.context -> |
|
77 |
Element.context_i list * Proof.context |
|
15596 | 78 |
|
79 |
(* Diagnostic functions *) |
|
12758 | 80 |
val print_locales: theory -> unit |
18137 | 81 |
val print_locale: theory -> bool -> expr -> Element.context list -> unit |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
82 |
val print_registrations: bool -> string -> Proof.context -> unit |
18137 | 83 |
|
27681 | 84 |
val add_locale: string -> bstring -> expr -> Element.context list -> theory |
20965 | 85 |
-> string * Proof.context |
27681 | 86 |
val add_locale_i: string -> bstring -> expr -> Element.context_i list -> theory |
20965 | 87 |
-> string * Proof.context |
15596 | 88 |
|
21225 | 89 |
(* Tactics *) |
90 |
val intro_locales_tac: bool -> Proof.context -> thm list -> tactic |
|
91 |
||
15696 | 92 |
(* Storing results *) |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
93 |
val add_thmss: string -> string -> (Attrib.binding * (thm list * Attrib.src list) list) list -> |
21582 | 94 |
Proof.context -> Proof.context |
24020 | 95 |
val add_type_syntax: string -> declaration -> Proof.context -> Proof.context |
96 |
val add_term_syntax: string -> declaration -> Proof.context -> Proof.context |
|
97 |
val add_declaration: string -> declaration -> Proof.context -> Proof.context |
|
18137 | 98 |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
99 |
val interpretation_i: (Proof.context -> Proof.context) -> |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
100 |
bool * string -> expr -> |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
101 |
term option list * (Attrib.binding * term) list -> |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
102 |
theory -> Proof.state |
21005 | 103 |
val interpretation: (Proof.context -> Proof.context) -> |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
104 |
bool * string -> expr -> |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
105 |
string option list * (Attrib.binding * string) list -> |
21005 | 106 |
theory -> Proof.state |
107 |
val interpretation_in_locale: (Proof.context -> Proof.context) -> |
|
108 |
xstring * expr -> theory -> Proof.state |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
109 |
val interpret_i: (Proof.state -> Proof.state Seq.seq) -> |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
110 |
bool * string -> expr -> |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
111 |
term option list * (Attrib.binding * term) list -> |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
112 |
bool -> Proof.state -> Proof.state |
21005 | 113 |
val interpret: (Proof.state -> Proof.state Seq.seq) -> |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
114 |
bool * string -> expr -> |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
115 |
string option list * (Attrib.binding * string) list -> |
21005 | 116 |
bool -> Proof.state -> Proof.state |
11896 | 117 |
end; |
12839 | 118 |
|
12289 | 119 |
structure Locale: LOCALE = |
11896 | 120 |
struct |
121 |
||
23228
05fb9b2b16d7
added gen_merge_lists/merge_lists/merge_alists (legacy operations from library.ML);
wenzelm
parents:
23178
diff
changeset
|
122 |
(* legacy operations *) |
05fb9b2b16d7
added gen_merge_lists/merge_lists/merge_alists (legacy operations from library.ML);
wenzelm
parents:
23178
diff
changeset
|
123 |
|
27681 | 124 |
fun merge_lists _ xs [] = xs |
125 |
| merge_lists _ [] ys = ys |
|
126 |
| merge_lists eq xs ys = xs @ filter_out (member eq xs) ys; |
|
127 |
||
128 |
fun merge_alists eq xs = merge_lists (eq_fst eq) xs; |
|
19780 | 129 |
|
20307 | 130 |
|
12273 | 131 |
(** locale elements and expressions **) |
11896 | 132 |
|
18137 | 133 |
datatype ctxt = datatype Element.ctxt; |
17355 | 134 |
|
12273 | 135 |
datatype expr = |
136 |
Locale of string | |
|
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
137 |
Rename of expr * (string * mixfix option) option list | |
12273 | 138 |
Merge of expr list; |
11896 | 139 |
|
12273 | 140 |
val empty = Merge []; |
141 |
||
18137 | 142 |
datatype 'a element = |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
143 |
Elem of 'a | Expr of expr; |
12273 | 144 |
|
18137 | 145 |
fun map_elem f (Elem e) = Elem (f e) |
146 |
| map_elem _ (Expr e) = Expr e; |
|
147 |
||
24020 | 148 |
type decl = declaration * stamp; |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
149 |
|
12070 | 150 |
type locale = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
151 |
{axiom: Element.witness list, |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
152 |
(* For locales that define predicates this is [A [A]], where A is the locale |
20317 | 153 |
specification. Otherwise []. |
154 |
Only required to generate the right witnesses for locales with predicates. *) |
|
19783 | 155 |
elems: (Element.context_i * stamp) list, |
156 |
(* Static content, neither Fixes nor Constrains elements *) |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
157 |
params: ((string * typ) * mixfix) list, (*all term params*) |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
158 |
decls: decl list * decl list, (*type/term_syntax declarations*) |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
159 |
regs: ((string * string list) * Element.witness list) list, |
19780 | 160 |
(* Registrations: indentifiers and witnesses of locales interpreted in the locale. *) |
25619 | 161 |
intros: thm list * thm list, |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
162 |
(* Introduction rules: of delta predicate and locale predicate. *) |
25619 | 163 |
dests: thm list} |
27761
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
164 |
(* Destruction rules: projections from locale predicate to predicates of fragments. *) |
11896 | 165 |
|
15703 | 166 |
(* CB: an internal (Int) locale element was either imported or included, |
167 |
an external (Ext) element appears directly in the locale text. *) |
|
168 |
||
169 |
datatype ('a, 'b) int_ext = Int of 'a | Ext of 'b; |
|
170 |
||
171 |
||
172 |
||
27761
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
173 |
(** substitutions on Vars -- clone from element.ML **) |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
174 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
175 |
(* instantiate types *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
176 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
177 |
fun var_instT_type env = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
178 |
if Vartab.is_empty env then I |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
179 |
else Term.map_type_tvar (fn (x, S) => the_default (TVar (x, S)) (Vartab.lookup env x)); |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
180 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
181 |
fun var_instT_term env = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
182 |
if Vartab.is_empty env then I |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
183 |
else Term.map_types (var_instT_type env); |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
184 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
185 |
fun var_inst_term (envT, env) = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
186 |
if Vartab.is_empty env then var_instT_term envT |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
187 |
else |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
188 |
let |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
189 |
val instT = var_instT_type envT; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
190 |
fun inst (Const (x, T)) = Const (x, instT T) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
191 |
| inst (Free (x, T)) = Free(x, instT T) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
192 |
| inst (Var (xi, T)) = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
193 |
(case Vartab.lookup env xi of |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
194 |
NONE => Var (xi, instT T) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
195 |
| SOME t => t) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
196 |
| inst (b as Bound _) = b |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
197 |
| inst (Abs (x, T, t)) = Abs (x, instT T, inst t) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
198 |
| inst (t $ u) = inst t $ inst u; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
199 |
in Envir.beta_norm o inst end; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
200 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
201 |
|
16736
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
202 |
(** management of registrations in theories and proof contexts **) |
11896 | 203 |
|
28005 | 204 |
type registration = |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
205 |
{prfx: (bool * string) * string, |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
206 |
(* first component: interpretation prefix; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
207 |
if the Boolean flag is set, only accesses containing the prefix are generated, |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
208 |
otherwise the prefix may be omitted when accessing theorems etc.) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
209 |
second component: parameter prefix *) |
28005 | 210 |
exp: Morphism.morphism, |
211 |
(* maps content to its originating context *) |
|
212 |
imp: (typ Vartab.table * typ list) * (term Vartab.table * term list), |
|
213 |
(* inverse of exp *) |
|
214 |
wits: Element.witness list, |
|
215 |
(* witnesses of the registration *) |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
216 |
eqns: thm Termtab.table, |
28005 | 217 |
(* theorems (equations) interpreting derived concepts and indexed by lhs *) |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
218 |
morph: unit |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
219 |
(* interpreting morphism *) |
28005 | 220 |
} |
221 |
||
15837 | 222 |
structure Registrations : |
223 |
sig |
|
224 |
type T |
|
225 |
val empty: T |
|
226 |
val join: T * T -> T |
|
20069
77a6b62418bb
Witness theorems of interpretations now transfered to current theory.
ballarin
parents:
20059
diff
changeset
|
227 |
val dest: theory -> T -> |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
228 |
(term list * |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
229 |
(((bool * string) * string) * |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
230 |
(Morphism.morphism * ((typ Vartab.table * typ list) * (term Vartab.table * term list))) * |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
231 |
Element.witness list * |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
232 |
thm Termtab.table)) list |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
233 |
val test: theory -> T * term list -> bool |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
234 |
val lookup: theory -> |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
235 |
T * (term list * ((typ Vartab.table * typ list) * (term Vartab.table * term list))) -> |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
236 |
(((bool * string) * string) * Element.witness list * thm Termtab.table) option |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
237 |
val insert: theory -> term list -> ((bool * string) * string) -> |
28005 | 238 |
(Morphism.morphism * ((typ Vartab.table * typ list) * (term Vartab.table * term list))) -> |
239 |
T -> |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
240 |
T * (term list * (((bool * string) * string) * Element.witness list)) list |
19780 | 241 |
val add_witness: term list -> Element.witness -> T -> T |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
242 |
val add_equation: term list -> thm -> T -> T |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
243 |
(* val update_morph: term list -> Element.witness list * thm list -> T -> T *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
244 |
(* val get_morph: theory -> T -> term list -> string list -> Morphism.morphism *) |
15837 | 245 |
end = |
246 |
struct |
|
28005 | 247 |
(* A registration is indexed by parameter instantiation. |
248 |
NB: index is exported whereas content is internalised. *) |
|
249 |
type T = registration Termtab.table; |
|
250 |
||
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
251 |
fun mk_reg prfx exp imp wits eqns morph = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
252 |
{prfx = prfx, exp = exp, imp = imp, wits = wits, eqns = eqns, morph = morph}; |
28005 | 253 |
|
254 |
fun map_reg f reg = |
|
255 |
let |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
256 |
val {prfx, exp, imp, wits, eqns, morph} = reg; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
257 |
val (prfx', exp', imp', wits', eqns', morph') = f (prfx, exp, imp, wits, eqns, morph); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
258 |
in mk_reg prfx' exp' imp' wits' eqns' morph' end; |
15837 | 259 |
|
260 |
val empty = Termtab.empty; |
|
261 |
||
262 |
(* term list represented as single term, for simultaneous matching *) |
|
263 |
fun termify ts = |
|
18343 | 264 |
Term.list_comb (Const ("", map fastype_of ts ---> propT), ts); |
15837 | 265 |
fun untermify t = |
266 |
let fun ut (Const _) ts = ts |
|
267 |
| ut (s $ t) ts = ut s (t::ts) |
|
268 |
in ut t [] end; |
|
269 |
||
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
270 |
(* joining of registrations: |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
271 |
- prefix and morphisms of right theory; |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
272 |
- witnesses are equal, no attempt to subsumption testing; |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
273 |
- union of equalities, if conflicting (i.e. two eqns with equal lhs) |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
274 |
eqn of right theory takes precedence *) |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
275 |
fun join (r1, r2) = Termtab.join (fn _ => fn ({eqns = e1, ...}, {prfx = n, exp, imp, wits = w, eqns = e2, morph = m}) => |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
276 |
mk_reg n exp imp w (Termtab.join (fn _ => fn (_, e) => e) (e1, e2)) m) (r1, r2); |
15837 | 277 |
|
20069
77a6b62418bb
Witness theorems of interpretations now transfered to current theory.
ballarin
parents:
20059
diff
changeset
|
278 |
fun dest_transfer thy regs = |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
279 |
Termtab.dest regs |> map (apsnd (map_reg (fn (n, e, i, ws, es, m) => |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
280 |
(n, e, i, map (Element.transfer_witness thy) ws, Termtab.map (transfer thy) es, m)))); |
28005 | 281 |
|
282 |
fun dest thy regs = dest_transfer thy regs |> map (apfst untermify) |> |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
283 |
map (apsnd (fn {prfx, exp, imp, wits, eqns, ...} => (prfx, (exp, imp), wits, eqns))); |
15837 | 284 |
|
285 |
(* registrations that subsume t *) |
|
17203 | 286 |
fun subsumers thy t regs = |
20069
77a6b62418bb
Witness theorems of interpretations now transfered to current theory.
ballarin
parents:
20059
diff
changeset
|
287 |
filter (fn (t', _) => Pattern.matches thy (t', t)) (dest_transfer thy regs); |
15837 | 288 |
|
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
289 |
(* test if registration that subsumes the query is present *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
290 |
fun test thy (regs, ts) = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
291 |
not (null (subsumers thy (termify ts) regs)); |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
292 |
|
15837 | 293 |
(* look up registration, pick one that subsumes the query *) |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
294 |
fun lookup thy (regs, (ts, ((impT, _), (imp, _)))) = |
15837 | 295 |
let |
296 |
val t = termify ts; |
|
19780 | 297 |
val subs = subsumers thy t regs; |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
298 |
in |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
299 |
(case subs of |
15837 | 300 |
[] => NONE |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
301 |
| ((t', {prfx, exp = exp', imp = ((impT', domT'), (imp', dom')), wits, eqns, morph}) :: _) => |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
302 |
let |
19780 | 303 |
val (tinst, inst) = Pattern.match thy (t', t) (Vartab.empty, Vartab.empty); |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
304 |
val tinst' = domT' |> map (fn (T as TFree (x, _)) => |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
305 |
(x, T |> Morphism.typ exp' |> Envir.typ_subst_TVars tinst |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
306 |
|> var_instT_type impT)) |> Symtab.make; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
307 |
val inst' = dom' |> map (fn (t as Free (x, _)) => |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
308 |
(x, t |> Morphism.term exp' |> Envir.subst_vars (tinst, inst) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
309 |
|> var_inst_term (impT, imp))) |> Symtab.make; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
310 |
val inst'_morph = Element.inst_morphism thy (tinst', inst'); |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
311 |
in SOME (prfx, |
28005 | 312 |
map (Element.morph_witness inst'_morph) wits, |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
313 |
Termtab.map (Morphism.thm inst'_morph) eqns) |
23918 | 314 |
end) |
15837 | 315 |
end; |
316 |
||
317 |
(* add registration if not subsumed by ones already present, |
|
318 |
additionally returns registrations that are strictly subsumed *) |
|
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
319 |
fun insert thy ts prfx (exp, imp) regs = |
15837 | 320 |
let |
321 |
val t = termify ts; |
|
20069
77a6b62418bb
Witness theorems of interpretations now transfered to current theory.
ballarin
parents:
20059
diff
changeset
|
322 |
val subs = subsumers thy t regs ; |
15837 | 323 |
in (case subs of |
324 |
[] => let |
|
325 |
val sups = |
|
20069
77a6b62418bb
Witness theorems of interpretations now transfered to current theory.
ballarin
parents:
20059
diff
changeset
|
326 |
filter (fn (t', _) => Pattern.matches thy (t, t')) (dest_transfer thy regs); |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
327 |
val sups' = map (apfst untermify) sups |> map (fn (ts, {prfx, wits, ...}) => (ts, (prfx, wits))) |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
328 |
in (Termtab.update (t, mk_reg prfx exp imp [] Termtab.empty ()) regs, sups') end |
15837 | 329 |
| _ => (regs, [])) |
330 |
end; |
|
331 |
||
25669 | 332 |
fun gen_add f ts regs = |
23918 | 333 |
let |
334 |
val t = termify ts; |
|
335 |
in |
|
28005 | 336 |
Termtab.update (t, map_reg f (the (Termtab.lookup regs t))) regs |
23918 | 337 |
end; |
338 |
||
15837 | 339 |
(* add witness theorem to registration, |
16169
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
340 |
only if instantiation is exact, otherwise exception Option raised *) |
25669 | 341 |
fun add_witness ts wit regs = |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
342 |
gen_add (fn (x, e, i, wits, eqns, m) => (x, e, i, Element.close_witness wit :: wits, eqns, m)) |
25669 | 343 |
ts regs; |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
344 |
|
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
345 |
(* add equation to registration, replaces previous equation with same lhs; |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
346 |
only if instantiation is exact, otherwise exception Option raised; |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
347 |
exception TERM raised if not a meta equality *) |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
348 |
fun add_equation ts thm regs = |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
349 |
gen_add (fn (x, e, i, thms, eqns, m) => |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
350 |
(x, e, i, thms, Termtab.update (thm |> prop_of |> Logic.dest_equals |> fst, Thm.close_derivation thm) eqns, m)) |
25669 | 351 |
ts regs; |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
352 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
353 |
(* update morphism of registration; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
354 |
only if instantiation is exact, otherwise exception Option raised *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
355 |
(* |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
356 |
fun update_morph ts (wits, eqns') regs = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
357 |
gen_add (fn (x, e, i, thms, eqns, _) => |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
358 |
(x, e, i, thms, eqns, (wits, eqns'))) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
359 |
ts regs; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
360 |
*) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
361 |
|
15837 | 362 |
end; |
363 |
||
16736
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
364 |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
365 |
(** theory data : locales **) |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
366 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
367 |
structure LocalesData = TheoryDataFun |
22846 | 368 |
( |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
369 |
type T = NameSpace.T * locale Symtab.table; |
15596 | 370 |
(* 1st entry: locale namespace, |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
371 |
2nd entry: locales of the theory *) |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
372 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
373 |
val empty = (NameSpace.empty, Symtab.empty); |
12063 | 374 |
val copy = I; |
16458 | 375 |
val extend = I; |
12289 | 376 |
|
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
377 |
fun join_locales _ |
27716 | 378 |
({axiom, elems, params, decls = (decls1, decls2), regs, intros, dests}: locale, |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
379 |
{elems = elems', decls = (decls1', decls2'), regs = regs', ...}: locale) = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
380 |
{axiom = axiom, |
27681 | 381 |
elems = merge_lists (eq_snd (op =)) elems elems', |
16736
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
382 |
params = params, |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
383 |
decls = |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
384 |
(Library.merge (eq_snd (op =)) (decls1, decls1'), |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
385 |
Library.merge (eq_snd (op =)) (decls2, decls2')), |
27681 | 386 |
regs = merge_alists (op =) regs regs', |
25619 | 387 |
intros = intros, |
388 |
dests = dests}; |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
389 |
fun merge _ ((space1, locs1), (space2, locs2)) = |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
390 |
(NameSpace.merge (space1, space2), Symtab.join join_locales (locs1, locs2)); |
22846 | 391 |
); |
15801 | 392 |
|
393 |
||
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
394 |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
395 |
(** context data : registrations **) |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
396 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
397 |
structure RegistrationsData = GenericDataFun |
22846 | 398 |
( |
399 |
type T = Registrations.T Symtab.table; (*registrations, indexed by locale name*) |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
400 |
val empty = Symtab.empty; |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
401 |
val extend = I; |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
402 |
fun merge _ = Symtab.join (K Registrations.join); |
22846 | 403 |
); |
12289 | 404 |
|
12277 | 405 |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
406 |
(** access locales **) |
12277 | 407 |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
408 |
val intern = NameSpace.intern o #1 o LocalesData.get; |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
409 |
val extern = NameSpace.extern o #1 o LocalesData.get; |
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
410 |
|
27681 | 411 |
fun get_locale thy name = Symtab.lookup (#2 (LocalesData.get thy)) name; |
412 |
||
413 |
fun the_locale thy name = case get_locale thy name |
|
414 |
of SOME loc => loc |
|
415 |
| NONE => error ("Unknown locale " ^ quote name); |
|
416 |
||
27686 | 417 |
fun register_locale name loc thy = |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
418 |
thy |> LocalesData.map (fn (space, locs) => |
27681 | 419 |
(Sign.declare_name thy name space, Symtab.update (name, loc) locs)); |
11896 | 420 |
|
18806 | 421 |
fun change_locale name f thy = |
422 |
let |
|
27716 | 423 |
val {axiom, elems, params, decls, regs, intros, dests} = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
424 |
the_locale thy name; |
27716 | 425 |
val (axiom', elems', params', decls', regs', intros', dests') = |
426 |
f (axiom, elems, params, decls, regs, intros, dests); |
|
18806 | 427 |
in |
27681 | 428 |
thy |
429 |
|> (LocalesData.map o apsnd) (Symtab.update (name, {axiom = axiom', |
|
27716 | 430 |
elems = elems', params = params', |
27681 | 431 |
decls = decls', regs = regs', intros = intros', dests = dests'})) |
432 |
end; |
|
433 |
||
434 |
fun print_locales thy = |
|
435 |
let val (space, locs) = LocalesData.get thy in |
|
436 |
Pretty.strs ("locales:" :: map #1 (NameSpace.extern_table (space, locs))) |
|
437 |
|> Pretty.writeln |
|
18806 | 438 |
end; |
439 |
||
12046 | 440 |
|
15596 | 441 |
(* access registrations *) |
442 |
||
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
443 |
(* retrieve registration from theory or context *) |
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
444 |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
445 |
fun get_registrations ctxt name = |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
446 |
case Symtab.lookup (RegistrationsData.get ctxt) name of |
15696 | 447 |
NONE => [] |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
448 |
| SOME reg => Registrations.dest (Context.theory_of ctxt) reg; |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
449 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
450 |
fun get_global_registrations thy = get_registrations (Context.Theory thy); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
451 |
fun get_local_registrations ctxt = get_registrations (Context.Proof ctxt); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
452 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
453 |
|
25357
6ea18fd11058
avoid "import" as identifier, which is a keyword in Alice;
wenzelm
parents:
25286
diff
changeset
|
454 |
fun get_registration ctxt imprt (name, ps) = |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
455 |
case Symtab.lookup (RegistrationsData.get ctxt) name of |
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
456 |
NONE => NONE |
25357
6ea18fd11058
avoid "import" as identifier, which is a keyword in Alice;
wenzelm
parents:
25286
diff
changeset
|
457 |
| SOME reg => Registrations.lookup (Context.theory_of ctxt) (reg, (ps, imprt)); |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
458 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
459 |
fun get_global_registration thy = get_registration (Context.Theory thy); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
460 |
fun get_local_registration ctxt = get_registration (Context.Proof ctxt); |
15596 | 461 |
|
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
462 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
463 |
fun test_registration ctxt (name, ps) = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
464 |
case Symtab.lookup (RegistrationsData.get ctxt) name of |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
465 |
NONE => false |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
466 |
| SOME reg => Registrations.test (Context.theory_of ctxt) (reg, ps); |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
467 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
468 |
fun test_global_registration thy = test_registration (Context.Theory thy); |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
469 |
fun test_local_registration ctxt = test_registration (Context.Proof ctxt); |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
470 |
|
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
471 |
|
15837 | 472 |
(* add registration to theory or context, ignored if subsumed *) |
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
473 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
474 |
fun put_registration (name, ps) prfx morphs ctxt = |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
475 |
RegistrationsData.map (fn regs => |
15837 | 476 |
let |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
477 |
val thy = Context.theory_of ctxt; |
18343 | 478 |
val reg = the_default Registrations.empty (Symtab.lookup regs name); |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
479 |
val (reg', sups) = Registrations.insert thy ps prfx morphs reg; |
15837 | 480 |
val _ = if not (null sups) then warning |
481 |
("Subsumed interpretation(s) of locale " ^ |
|
16458 | 482 |
quote (extern thy name) ^ |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
483 |
"\nwith the following prefix(es):" ^ |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
484 |
commas_quote (map (fn (_, ((_, s), _)) => s) sups)) |
15837 | 485 |
else (); |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
486 |
in Symtab.update (name, reg') regs end) ctxt; |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
487 |
|
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
488 |
fun put_global_registration id prfx morphs = |
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
489 |
Context.theory_map (put_registration id prfx morphs); |
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
490 |
fun put_local_registration id prfx morphs = |
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
491 |
Context.proof_map (put_registration id prfx morphs); |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
492 |
|
15596 | 493 |
|
18806 | 494 |
fun put_registration_in_locale name id = |
27716 | 495 |
change_locale name (fn (axiom, elems, params, decls, regs, intros, dests) => |
496 |
(axiom, elems, params, decls, regs @ [(id, [])], intros, dests)); |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
497 |
|
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
498 |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
499 |
(* add witness theorem to registration, ignored if registration not present *) |
15596 | 500 |
|
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
501 |
fun add_witness (name, ps) thm = |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
502 |
RegistrationsData.map (Symtab.map_entry name (Registrations.add_witness ps thm)); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
503 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
504 |
fun add_global_witness id thm = Context.theory_map (add_witness id thm); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
505 |
fun add_local_witness id thm = Context.proof_map (add_witness id thm); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
506 |
|
15596 | 507 |
|
18806 | 508 |
fun add_witness_in_locale name id thm = |
27716 | 509 |
change_locale name (fn (axiom, elems, params, decls, regs, intros, dests) => |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
510 |
let |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
511 |
fun add (id', thms) = |
18806 | 512 |
if id = id' then (id', thm :: thms) else (id', thms); |
27716 | 513 |
in (axiom, elems, params, decls, map add regs, intros, dests) end); |
15596 | 514 |
|
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
515 |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
516 |
(* add equation to registration, ignored if registration not present *) |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
517 |
|
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
518 |
fun add_equation (name, ps) thm = |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
519 |
RegistrationsData.map (Symtab.map_entry name (Registrations.add_equation ps thm)); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
520 |
|
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
521 |
fun add_global_equation id thm = Context.theory_map (add_equation id thm); |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
522 |
fun add_local_equation id thm = Context.proof_map (add_equation id thm); |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
523 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
524 |
(* |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
525 |
(* update morphism of registration, ignored if registration not present *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
526 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
527 |
fun update_morph (name, ps) morph = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
528 |
RegistrationsData.map (Symtab.map_entry name (Registrations.update_morph ps morph)); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
529 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
530 |
fun update_global_morph id morph = Context.theory_map (update_morph id morph); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
531 |
fun update_local_morph id morph = Context.proof_map (update_morph id morph); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
532 |
*) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
533 |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
534 |
|
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
535 |
(* printing of registrations *) |
15596 | 536 |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
537 |
fun print_registrations show_wits loc ctxt = |
15596 | 538 |
let |
15703 | 539 |
val thy = ProofContext.theory_of ctxt; |
24920 | 540 |
val prt_term = Pretty.quote o Syntax.pretty_term ctxt; |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
541 |
fun prt_term' t = if !show_types |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
542 |
then Pretty.block [prt_term t, Pretty.brk 1, Pretty.str "::", |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
543 |
Pretty.brk 1, (Pretty.quote o Syntax.pretty_typ ctxt) (type_of t)] |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
544 |
else prt_term t; |
23918 | 545 |
val prt_thm = prt_term o prop_of; |
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
546 |
fun prt_inst ts = |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
547 |
Pretty.enclose "(" ")" (Pretty.breaks (map prt_term' ts)); |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
548 |
fun prt_prfx ((false, prfx), pprfx) = [Pretty.str prfx, Pretty.brk 1, Pretty.str "(optional)", Pretty.brk 1, Pretty.str pprfx] |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
549 |
| prt_prfx ((true, prfx), pprfx) = [Pretty.str prfx, Pretty.brk 1, Pretty.str pprfx]; |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
550 |
fun prt_eqns [] = Pretty.str "no equations." |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
551 |
| prt_eqns eqns = Pretty.block (Pretty.str "equations:" :: Pretty.brk 1 :: |
23918 | 552 |
Pretty.breaks (map prt_thm eqns)); |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
553 |
fun prt_core ts eqns = |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
554 |
[prt_inst ts, Pretty.fbrk, prt_eqns (Termtab.dest eqns |> map snd)]; |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
555 |
fun prt_witns [] = Pretty.str "no witnesses." |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
556 |
| prt_witns witns = Pretty.block (Pretty.str "witnesses:" :: Pretty.brk 1 :: |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
557 |
Pretty.breaks (map (Element.pretty_witness ctxt) witns)) |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
558 |
fun prt_reg (ts, ((_, ""), _, witns, eqns)) = |
17138 | 559 |
if show_wits |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
560 |
then Pretty.block (prt_core ts eqns @ [Pretty.fbrk, prt_witns witns]) |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
561 |
else Pretty.block (prt_core ts eqns) |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
562 |
| prt_reg (ts, (prfx, _, witns, eqns)) = |
17138 | 563 |
if show_wits |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
564 |
then Pretty.block ((prt_prfx prfx @ [Pretty.str ":", Pretty.brk 1] @ |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
565 |
prt_core ts eqns @ [Pretty.fbrk, prt_witns witns])) |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
566 |
else Pretty.block ((prt_prfx prfx @ |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
567 |
[Pretty.str ":", Pretty.brk 1] @ prt_core ts eqns)); |
15703 | 568 |
|
16458 | 569 |
val loc_int = intern thy loc; |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
570 |
val regs = RegistrationsData.get (Context.Proof ctxt); |
17412 | 571 |
val loc_regs = Symtab.lookup regs loc_int; |
15596 | 572 |
in |
573 |
(case loc_regs of |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
574 |
NONE => Pretty.str ("no interpretations") |
15763
b901a127ac73
Interpretation supports statically scoped attributes; documentation.
ballarin
parents:
15749
diff
changeset
|
575 |
| SOME r => let |
20069
77a6b62418bb
Witness theorems of interpretations now transfered to current theory.
ballarin
parents:
20059
diff
changeset
|
576 |
val r' = Registrations.dest thy r; |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
577 |
val r'' = Library.sort_wrt (fn (_, ((_, prfx), _, _, _)) => prfx) r'; |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
578 |
in Pretty.big_list ("interpretations:") (map prt_reg r'') end) |
15596 | 579 |
|> Pretty.writeln |
580 |
end; |
|
581 |
||
582 |
||
12277 | 583 |
(* diagnostics *) |
12273 | 584 |
|
12277 | 585 |
fun err_in_locale ctxt msg ids = |
586 |
let |
|
16458 | 587 |
val thy = ProofContext.theory_of ctxt; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
588 |
fun prt_id (name, parms) = |
16458 | 589 |
[Pretty.block (Pretty.breaks (map Pretty.str (extern thy name :: parms)))]; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
590 |
val prt_ids = flat (separate [Pretty.str " +", Pretty.brk 1] (map prt_id ids)); |
12502 | 591 |
val err_msg = |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
592 |
if forall (equal "" o #1) ids then msg |
12502 | 593 |
else msg ^ "\n" ^ Pretty.string_of (Pretty.block |
594 |
(Pretty.str "The error(s) above occurred in locale:" :: Pretty.brk 1 :: prt_ids)); |
|
18678 | 595 |
in error err_msg end; |
12063 | 596 |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
597 |
fun err_in_locale' ctxt msg ids' = err_in_locale ctxt msg (map fst ids'); |
12277 | 598 |
|
599 |
||
19783 | 600 |
fun pretty_ren NONE = Pretty.str "_" |
601 |
| pretty_ren (SOME (x, NONE)) = Pretty.str x |
|
602 |
| pretty_ren (SOME (x, SOME syn)) = |
|
603 |
Pretty.block [Pretty.str x, Pretty.brk 1, Syntax.pretty_mixfix syn]; |
|
604 |
||
605 |
fun pretty_expr thy (Locale name) = Pretty.str (extern thy name) |
|
606 |
| pretty_expr thy (Rename (expr, xs)) = |
|
607 |
Pretty.block [pretty_expr thy expr, Pretty.brk 1, Pretty.block (map pretty_ren xs |> Pretty.breaks)] |
|
608 |
| pretty_expr thy (Merge es) = |
|
609 |
Pretty.separate "+" (map (pretty_expr thy) es) |> Pretty.block; |
|
610 |
||
611 |
fun err_in_expr _ msg (Merge []) = error msg |
|
612 |
| err_in_expr ctxt msg expr = |
|
613 |
error (msg ^ "\n" ^ Pretty.string_of (Pretty.block |
|
614 |
[Pretty.str "The error(s) above occured in locale expression:", Pretty.brk 1, |
|
615 |
pretty_expr (ProofContext.theory_of ctxt) expr])); |
|
616 |
||
12046 | 617 |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
618 |
(** structured contexts: rename + merge + implicit type instantiation **) |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
619 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
620 |
(* parameter types *) |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
621 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
622 |
fun frozen_tvars ctxt Ts = |
19914 | 623 |
#1 (Variable.importT_inst (map Logic.mk_type Ts) ctxt) |
19900
21a99d88d925
ProofContext: moved variable operations to struct Variable;
wenzelm
parents:
19873
diff
changeset
|
624 |
|> map (fn ((xi, S), T) => (xi, (S, T))); |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
625 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
626 |
fun unify_frozen ctxt maxidx Ts Us = |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
627 |
let |
18343 | 628 |
fun paramify NONE i = (NONE, i) |
629 |
| paramify (SOME T) i = apfst SOME (TypeInfer.paramify_dummies T i); |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
630 |
|
18343 | 631 |
val (Ts', maxidx') = fold_map paramify Ts maxidx; |
632 |
val (Us', maxidx'') = fold_map paramify Us maxidx'; |
|
16947 | 633 |
val thy = ProofContext.theory_of ctxt; |
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
634 |
|
18190 | 635 |
fun unify (SOME T, SOME U) env = (Sign.typ_unify thy (U, T) env |
636 |
handle Type.TUNIFY => raise TYPE ("unify_frozen: failed to unify types", [U, T], [])) |
|
637 |
| unify _ env = env; |
|
638 |
val (unifier, _) = fold unify (Ts' ~~ Us') (Vartab.empty, maxidx''); |
|
15570 | 639 |
val Vs = map (Option.map (Envir.norm_type unifier)) Us'; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
640 |
val unifier' = Vartab.extend (unifier, frozen_tvars ctxt (map_filter I Vs)); |
15570 | 641 |
in map (Option.map (Envir.norm_type unifier')) Vs end; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
642 |
|
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
643 |
fun params_of elemss = |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
644 |
distinct (eq_fst (op = : string * string -> bool)) (maps (snd o fst) elemss); |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
645 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
646 |
fun params_of' elemss = |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
647 |
distinct (eq_fst (op = : string * string -> bool)) (maps (snd o fst o fst) elemss); |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
648 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
649 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
650 |
fun param_prefix params = space_implode "_" params; |
26645
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
651 |
fun params_qualified params name = |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
652 |
NameSpace.qualified (param_prefix params) name; |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
653 |
|
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
654 |
|
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
655 |
(* CB: param_types has the following type: |
15531 | 656 |
('a * 'b option) list -> ('a * 'b) list *) |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
657 |
fun param_types ps = map_filter (fn (_, NONE) => NONE | (x, SOME T) => SOME (x, T)) ps; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
658 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
659 |
|
19932 | 660 |
fun merge_syntax ctxt ids ss = Symtab.merge (op = : mixfix * mixfix -> bool) ss |
23655
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm
parents:
23591
diff
changeset
|
661 |
handle Symtab.DUP x => err_in_locale ctxt |
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm
parents:
23591
diff
changeset
|
662 |
("Conflicting syntax for parameter: " ^ quote x) (map fst ids); |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
663 |
|
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
664 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
665 |
(* Distinction of assumed vs. derived identifiers. |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
666 |
The former may have axioms relating assumptions of the context to |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
667 |
assumptions of the specification fragment (for locales with |
19780 | 668 |
predicates). The latter have witnesses relating assumptions of the |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
669 |
specification fragment to assumptions of other (assumed) specification |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
670 |
fragments. *) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
671 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
672 |
datatype 'a mode = Assumed of 'a | Derived of 'a; |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
673 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
674 |
fun map_mode f (Assumed x) = Assumed (f x) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
675 |
| map_mode f (Derived x) = Derived (f x); |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
676 |
|
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
677 |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
678 |
(* flatten expressions *) |
11896 | 679 |
|
12510 | 680 |
local |
12502 | 681 |
|
18137 | 682 |
fun unify_parms ctxt fixed_parms raw_parmss = |
12502 | 683 |
let |
16458 | 684 |
val thy = ProofContext.theory_of ctxt; |
12502 | 685 |
val maxidx = length raw_parmss; |
686 |
val idx_parmss = (0 upto maxidx - 1) ~~ raw_parmss; |
|
687 |
||
688 |
fun varify i = Term.map_type_tfree (fn (a, S) => TVar ((a, i), S)); |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
689 |
fun varify_parms (i, ps) = map (apsnd (varify i)) (param_types ps); |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
690 |
val parms = fixed_parms @ maps varify_parms idx_parmss; |
12502 | 691 |
|
18137 | 692 |
fun unify T U envir = Sign.typ_unify thy (U, T) envir |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
693 |
handle Type.TUNIFY => |
23418 | 694 |
let |
22339
0dc6b45e5662
more precise error message in parameter unification
schirmer
parents:
22300
diff
changeset
|
695 |
val T' = Envir.norm_type (fst envir) T; |
0dc6b45e5662
more precise error message in parameter unification
schirmer
parents:
22300
diff
changeset
|
696 |
val U' = Envir.norm_type (fst envir) U; |
26948 | 697 |
val prt = Syntax.string_of_typ ctxt; |
22339
0dc6b45e5662
more precise error message in parameter unification
schirmer
parents:
22300
diff
changeset
|
698 |
in |
18137 | 699 |
raise TYPE ("unify_parms: failed to unify types " ^ |
22339
0dc6b45e5662
more precise error message in parameter unification
schirmer
parents:
22300
diff
changeset
|
700 |
prt U' ^ " and " ^ prt T', [U', T'], []) |
18137 | 701 |
end; |
702 |
fun unify_list (T :: Us) = fold (unify T) Us |
|
703 |
| unify_list [] = I; |
|
18952 | 704 |
val (unifier, _) = fold unify_list (map #2 (Symtab.dest (Symtab.make_list parms))) |
18137 | 705 |
(Vartab.empty, maxidx); |
12502 | 706 |
|
19061
ffbbac0261c9
removed distinct, renamed gen_distinct to distinct;
wenzelm
parents:
19025
diff
changeset
|
707 |
val parms' = map (apsnd (Envir.norm_type unifier)) (distinct (eq_fst (op =)) parms); |
12502 | 708 |
val unifier' = Vartab.extend (unifier, frozen_tvars ctxt (map #2 parms')); |
709 |
||
710 |
fun inst_parms (i, ps) = |
|
23178 | 711 |
List.foldr Term.add_typ_tfrees [] (map_filter snd ps) |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
712 |
|> map_filter (fn (a, S) => |
12502 | 713 |
let val T = Envir.norm_type unifier' (TVar ((a, i), S)) |
18137 | 714 |
in if T = TFree (a, S) then NONE else SOME (a, T) end) |
715 |
|> Symtab.make; |
|
716 |
in map inst_parms idx_parmss end; |
|
12502 | 717 |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
718 |
in |
12502 | 719 |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
720 |
fun unify_elemss _ _ [] = [] |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
721 |
| unify_elemss _ [] [elems] = [elems] |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
722 |
| unify_elemss ctxt fixed_parms elemss = |
12502 | 723 |
let |
18137 | 724 |
val thy = ProofContext.theory_of ctxt; |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
725 |
val phis = unify_parms ctxt fixed_parms (map (snd o fst o fst) elemss) |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
726 |
|> map (Element.instT_morphism thy); |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
727 |
fun inst ((((name, ps), mode), elems), phi) = |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
728 |
(((name, map (apsnd (Option.map (Morphism.typ phi))) ps), |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
729 |
map_mode (map (Element.morph_witness phi)) mode), |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
730 |
map (Element.morph_ctxt phi) elems); |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
731 |
in map inst (elemss ~~ phis) end; |
12502 | 732 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
733 |
|
19810 | 734 |
fun renaming xs parms = zip_options parms xs |
735 |
handle Library.UnequalLengths => |
|
736 |
error ("Too many arguments in renaming: " ^ |
|
737 |
commas (map (fn NONE => "_" | SOME x => quote (fst x)) xs)); |
|
738 |
||
739 |
||
19783 | 740 |
(* params_of_expr: |
741 |
Compute parameters (with types and syntax) of locale expression. |
|
742 |
*) |
|
743 |
||
744 |
fun params_of_expr ctxt fixed_params expr (prev_parms, prev_types, prev_syn) = |
|
745 |
let |
|
746 |
val thy = ProofContext.theory_of ctxt; |
|
747 |
||
748 |
fun merge_tenvs fixed tenv1 tenv2 = |
|
749 |
let |
|
750 |
val [env1, env2] = unify_parms ctxt fixed |
|
751 |
[tenv1 |> Symtab.dest |> map (apsnd SOME), |
|
752 |
tenv2 |> Symtab.dest |> map (apsnd SOME)] |
|
753 |
in |
|
754 |
Symtab.merge (op =) (Symtab.map (Element.instT_type env1) tenv1, |
|
755 |
Symtab.map (Element.instT_type env2) tenv2) |
|
756 |
end; |
|
757 |
||
758 |
fun merge_syn expr syn1 syn2 = |
|
19932 | 759 |
Symtab.merge (op = : mixfix * mixfix -> bool) (syn1, syn2) |
23655
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm
parents:
23591
diff
changeset
|
760 |
handle Symtab.DUP x => err_in_expr ctxt |
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm
parents:
23591
diff
changeset
|
761 |
("Conflicting syntax for parameter: " ^ quote x) expr; |
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
762 |
|
19783 | 763 |
fun params_of (expr as Locale name) = |
764 |
let |
|
27716 | 765 |
val {params, ...} = the_locale thy name; |
766 |
in (map (fst o fst) params, params |> map fst |> Symtab.make, |
|
767 |
params |> map (apfst fst) |> Symtab.make) end |
|
19783 | 768 |
| params_of (expr as Rename (e, xs)) = |
769 |
let |
|
770 |
val (parms', types', syn') = params_of e; |
|
771 |
val ren = renaming xs parms'; |
|
772 |
(* renaming may reduce number of parameters *) |
|
773 |
val new_parms = map (Element.rename ren) parms' |> distinct (op =); |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
774 |
val ren_syn = syn' |> Symtab.dest |> map (Element.rename_var_name ren); |
19783 | 775 |
val new_syn = fold (Symtab.insert (op =)) ren_syn Symtab.empty |
776 |
handle Symtab.DUP x => |
|
777 |
err_in_expr ctxt ("Conflicting syntax for parameter: " ^ quote x) expr; |
|
22700 | 778 |
val syn_types = map (apsnd (fn mx => |
779 |
SOME (Type.freeze_type (#1 (TypeInfer.paramify_dummies (Syntax.mixfixT mx) 0))))) |
|
780 |
(Symtab.dest new_syn); |
|
19783 | 781 |
val ren_types = types' |> Symtab.dest |> map (apfst (Element.rename ren)); |
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
782 |
val (env :: _) = unify_parms ctxt [] |
19783 | 783 |
((ren_types |> map (apsnd SOME)) :: map single syn_types); |
784 |
val new_types = fold (Symtab.insert (op =)) |
|
785 |
(map (apsnd (Element.instT_type env)) ren_types) Symtab.empty; |
|
786 |
in (new_parms, new_types, new_syn) end |
|
787 |
| params_of (Merge es) = |
|
788 |
fold (fn e => fn (parms, types, syn) => |
|
789 |
let |
|
790 |
val (parms', types', syn') = params_of e |
|
791 |
in |
|
27681 | 792 |
(merge_lists (op =) parms parms', merge_tenvs [] types types', |
19783 | 793 |
merge_syn e syn syn') |
794 |
end) |
|
795 |
es ([], Symtab.empty, Symtab.empty) |
|
796 |
||
797 |
val (parms, types, syn) = params_of expr; |
|
798 |
in |
|
27681 | 799 |
(merge_lists (op =) prev_parms parms, merge_tenvs fixed_params prev_types types, |
19783 | 800 |
merge_syn expr prev_syn syn) |
801 |
end; |
|
802 |
||
803 |
fun make_params_ids params = [(("", params), ([], Assumed []))]; |
|
804 |
fun make_raw_params_elemss (params, tenv, syn) = |
|
805 |
[((("", map (fn p => (p, Symtab.lookup tenv p)) params), Assumed []), |
|
806 |
Int [Fixes (map (fn p => |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
807 |
(Name.binding p, Symtab.lookup tenv p, Symtab.lookup syn p |> the)) params)])]; |
19783 | 808 |
|
809 |
||
15596 | 810 |
(* flatten_expr: |
811 |
Extend list of identifiers by those new in locale expression expr. |
|
812 |
Compute corresponding list of lists of locale elements (one entry per |
|
813 |
identifier). |
|
814 |
||
815 |
Identifiers represent locale fragments and are in an extended form: |
|
816 |
((name, ps), (ax_ps, axs)) |
|
817 |
(name, ps) is the locale name with all its parameters. |
|
818 |
(ax_ps, axs) is the locale axioms with its parameters; |
|
819 |
axs are always taken from the top level of the locale hierarchy, |
|
820 |
hence axioms may contain additional parameters from later fragments: |
|
821 |
ps subset of ax_ps. axs is either singleton or empty. |
|
822 |
||
823 |
Elements are enriched by identifier-like information: |
|
824 |
(((name, ax_ps), axs), elems) |
|
825 |
The parameters in ax_ps are the axiom parameters, but enriched by type |
|
826 |
info: now each entry is a pair of string and typ option. Axioms are |
|
827 |
type-instantiated. |
|
828 |
||
829 |
*) |
|
830 |
||
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
831 |
fun flatten_expr ctxt ((prev_idents, prev_syntax), expr) = |
12014 | 832 |
let |
833 |
val thy = ProofContext.theory_of ctxt; |
|
12263 | 834 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
835 |
fun rename_parms top ren ((name, ps), (parms, mode)) = |
19783 | 836 |
((name, map (Element.rename ren) ps), |
837 |
if top |
|
838 |
then (map (Element.rename ren) parms, |
|
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
839 |
map_mode (map (Element.morph_witness (Element.rename_morphism ren))) mode) |
19783 | 840 |
else (parms, mode)); |
12263 | 841 |
|
27716 | 842 |
(* add (name, pTs) and its registrations, recursively; adjust hyps of witnesses *) |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
843 |
|
20167
fe5fd4fd4114
Strict dfs traversal of imported and registered identifiers.
ballarin
parents:
20092
diff
changeset
|
844 |
fun add_with_regs ((name, pTs), mode) (wits, ids, visited) = |
fe5fd4fd4114
Strict dfs traversal of imported and registered identifiers.
ballarin
parents:
20092
diff
changeset
|
845 |
if member (fn (a, (b, _)) => a = b) visited (name, map #1 pTs) |
fe5fd4fd4114
Strict dfs traversal of imported and registered identifiers.
ballarin
parents:
20092
diff
changeset
|
846 |
then (wits, ids, visited) |
fe5fd4fd4114
Strict dfs traversal of imported and registered identifiers.
ballarin
parents:
20092
diff
changeset
|
847 |
else |
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
848 |
let |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
849 |
val {params, regs, ...} = the_locale thy name; |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
850 |
val pTs' = map #1 params; |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
851 |
val ren = map #1 pTs' ~~ map (fn (x, _) => (x, NONE)) pTs; |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
852 |
(* dummy syntax, since required by rename *) |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
853 |
val pTs'' = map (fn ((p, _), (_, T)) => (p, T)) (pTs ~~ pTs'); |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
854 |
val [env] = unify_parms ctxt pTs [map (apsnd SOME) pTs'']; |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
855 |
(* propagate parameter types, to keep them consistent *) |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
856 |
val regs' = map (fn ((name, ps), wits) => |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
857 |
((name, map (Element.rename ren) ps), |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
858 |
map (Element.transfer_witness thy) wits)) regs; |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
859 |
val new_regs = regs'; |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
860 |
val new_ids = map fst new_regs; |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
861 |
val new_idTs = |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
862 |
map (apsnd (map (fn p => (p, (the o AList.lookup (op =) pTs) p)))) new_ids; |
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
863 |
|
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
864 |
val new_wits = new_regs |> map (#2 #> map |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
865 |
(Element.morph_witness |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
866 |
(Element.instT_morphism thy env $> |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
867 |
Element.rename_morphism ren $> |
25669 | 868 |
Element.satisfy_morphism wits) |
869 |
#> Element.close_witness)); |
|
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
870 |
val new_ids' = map (fn (id, wits) => |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
871 |
(id, ([], Derived wits))) (new_ids ~~ new_wits); |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
872 |
val new_idTs' = map (fn ((n, pTs), (_, ([], mode))) => |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
873 |
((n, pTs), mode)) (new_idTs ~~ new_ids'); |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
874 |
val new_id = ((name, map #1 pTs), ([], mode)); |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
875 |
val (wits', ids', visited') = fold add_with_regs new_idTs' |
20167
fe5fd4fd4114
Strict dfs traversal of imported and registered identifiers.
ballarin
parents:
20092
diff
changeset
|
876 |
(wits @ flat new_wits, ids, visited @ [new_id]); |
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
877 |
in |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
878 |
(wits', ids' @ [new_id], visited') |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
879 |
end; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
880 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
881 |
(* distribute top-level axioms over assumed ids *) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
882 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
883 |
fun axiomify all_ps ((name, parms), (_, Assumed _)) axioms = |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
884 |
let |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
885 |
val {elems, ...} = the_locale thy name; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
886 |
val ts = maps |
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
887 |
(fn (Assumes asms, _) => maps (map #1 o #2) asms |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
888 |
| _ => []) |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
889 |
elems; |
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
890 |
val (axs1, axs2) = chop (length ts) axioms; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
891 |
in (((name, parms), (all_ps, Assumed axs1)), axs2) end |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
892 |
| axiomify all_ps (id, (_, Derived ths)) axioms = |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
893 |
((id, (all_ps, Derived ths)), axioms); |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
894 |
|
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
895 |
(* identifiers of an expression *) |
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
896 |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
897 |
fun identify top (Locale name) = |
15596 | 898 |
(* CB: ids_ax is a list of tuples of the form ((name, ps), axs), |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
899 |
where name is a locale name, ps a list of parameter names and axs |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
900 |
a list of axioms relating to the identifier, axs is empty unless |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
901 |
identify at top level (top = true); |
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
902 |
parms is accumulated list of parameters *) |
12289 | 903 |
let |
27716 | 904 |
val {axiom, params, ...} = the_locale thy name; |
19278 | 905 |
val ps = map (#1 o #1) params; |
27716 | 906 |
val (_, ids'', _) = add_with_regs ((name, map #1 params), Assumed []) ([], [], []); |
20167
fe5fd4fd4114
Strict dfs traversal of imported and registered identifiers.
ballarin
parents:
20092
diff
changeset
|
907 |
val ids_ax = if top then fst (fold_map (axiomify ps) ids'' axiom) else ids''; |
27716 | 908 |
in (ids_ax, ps) end |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
909 |
| identify top (Rename (e, xs)) = |
12273 | 910 |
let |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
911 |
val (ids', parms') = identify top e; |
12839 | 912 |
val ren = renaming xs parms' |
18678 | 913 |
handle ERROR msg => err_in_locale' ctxt msg ids'; |
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
914 |
|
19061
ffbbac0261c9
removed distinct, renamed gen_distinct to distinct;
wenzelm
parents:
19025
diff
changeset
|
915 |
val ids'' = distinct (eq_fst (op =)) (map (rename_parms top ren) ids'); |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
916 |
val parms'' = distinct (op =) (maps (#2 o #1) ids''); |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
917 |
in (ids'', parms'') end |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
918 |
| identify top (Merge es) = |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
919 |
fold (fn e => fn (ids, parms) => |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
920 |
let |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
921 |
val (ids', parms') = identify top e |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
922 |
in |
27681 | 923 |
(merge_alists (op =) ids ids', merge_lists (op =) parms parms') |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
924 |
end) |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
925 |
es ([], []); |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
926 |
|
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
927 |
fun inst_wit all_params (t, th) = let |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
928 |
val {hyps, prop, ...} = Thm.rep_thm th; |
16861 | 929 |
val ps = map (apsnd SOME) (fold Term.add_frees (prop :: hyps) []); |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
930 |
val [env] = unify_parms ctxt all_params [ps]; |
18137 | 931 |
val t' = Element.instT_term env t; |
932 |
val th' = Element.instT_thm thy env th; |
|
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
933 |
in (t', th') end; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
934 |
|
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
935 |
fun eval all_params tenv syn ((name, params), (locale_params, mode)) = |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
936 |
let |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
937 |
val {params = ps_mx, elems = elems_stamped, ...} = the_locale thy name; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
938 |
val elems = map fst elems_stamped; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
939 |
val ps = map fst ps_mx; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
940 |
fun lookup_syn x = (case Symtab.lookup syn x of SOME Structure => NONE | opt => opt); |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
941 |
val locale_params' = map (fn p => (p, Symtab.lookup tenv p |> the)) locale_params; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
942 |
val mode' = map_mode (map (Element.map_witness (inst_wit all_params))) mode; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
943 |
val ren = map fst ps ~~ map (fn p => (p, lookup_syn p)) params; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
944 |
val [env] = unify_parms ctxt all_params [map (apfst (Element.rename ren) o apsnd SOME) ps]; |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
945 |
val elem_morphism = |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
946 |
Element.rename_morphism ren $> |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
947 |
Morphism.name_morphism (Name.map_name (params_qualified params)) $> |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
948 |
Element.instT_morphism thy env; |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
949 |
val elems' = map (Element.morph_ctxt elem_morphism) elems; |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
950 |
in (((name, map (apsnd SOME) locale_params'), mode'), elems') end; |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
951 |
|
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
952 |
(* parameters, their types and syntax *) |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
953 |
val (all_params', tenv, syn) = params_of_expr ctxt [] expr ([], Symtab.empty, Symtab.empty); |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
954 |
val all_params = map (fn p => (p, Symtab.lookup tenv p |> the)) all_params'; |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
955 |
(* compute identifiers and syntax, merge with previous ones *) |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
956 |
val (ids, _) = identify true expr; |
20951
868120282837
gen_rem(s) abandoned in favour of remove / subtract
haftmann
parents:
20911
diff
changeset
|
957 |
val idents = subtract (eq_fst (op =)) prev_idents ids; |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
958 |
val syntax = merge_syntax ctxt ids (syn, prev_syntax); |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
959 |
(* type-instantiate elements *) |
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
960 |
val final_elemss = map (eval all_params tenv syntax) idents; |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
961 |
in ((prev_idents @ idents, syntax), final_elemss) end; |
12046 | 962 |
|
12510 | 963 |
end; |
964 |
||
12070 | 965 |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
966 |
(* activate elements *) |
12273 | 967 |
|
12510 | 968 |
local |
969 |
||
21686 | 970 |
fun axioms_export axs _ As = |
971 |
(Element.satisfy_thm axs #> Drule.implies_intr_list (Library.drop (length axs, As)), fn t => t); |
|
12263 | 972 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
973 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
974 |
(* NB: derived ids contain only facts at this stage *) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
975 |
|
27681 | 976 |
fun activate_elem _ _ (Fixes fixes) (ctxt, mode) = |
977 |
([], (ctxt |> ProofContext.add_fixes_i fixes |> snd, mode)) |
|
978 |
| activate_elem _ _ (Constrains _) (ctxt, mode) = |
|
979 |
([], (ctxt, mode)) |
|
980 |
| activate_elem ax_in_ctxt _ (Assumes asms) (ctxt, Assumed axs) = |
|
13399
c136276dc847
support locale ``views'' (for cumulative predicates);
wenzelm
parents:
13394
diff
changeset
|
981 |
let |
18728 | 982 |
val asms' = Attrib.map_specs (Attrib.attribute_i (ProofContext.theory_of ctxt)) asms; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
983 |
val ts = maps (map #1 o #2) asms'; |
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
984 |
val (ps, qs) = chop (length ts) axs; |
17856 | 985 |
val (_, ctxt') = |
21370
d9dd7b4e5e69
replaced Variable.fix_frees by Variable.auto_fixes (depends on body mode);
wenzelm
parents:
21361
diff
changeset
|
986 |
ctxt |> fold Variable.auto_fixes ts |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
987 |
|> ProofContext.add_assms_i (axioms_export (if ax_in_ctxt then ps else [])) asms'; |
27681 | 988 |
in ([], (ctxt', Assumed qs)) end |
989 |
| activate_elem _ _ (Assumes asms) (ctxt, Derived ths) = |
|
990 |
([], (ctxt, Derived ths)) |
|
991 |
| activate_elem _ _ (Defines defs) (ctxt, Assumed axs) = |
|
15596 | 992 |
let |
18728 | 993 |
val defs' = Attrib.map_specs (Attrib.attribute_i (ProofContext.theory_of ctxt)) defs; |
19732 | 994 |
val asms = defs' |> map (fn ((name, atts), (t, ps)) => |
995 |
let val ((c, _), t') = LocalDefs.cert_def ctxt t |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
996 |
in (t', ((Name.map_name (Thm.def_name_optional c) name, atts), [(t', ps)])) end); |
17856 | 997 |
val (_, ctxt') = |
21370
d9dd7b4e5e69
replaced Variable.fix_frees by Variable.auto_fixes (depends on body mode);
wenzelm
parents:
21361
diff
changeset
|
998 |
ctxt |> fold (Variable.auto_fixes o #1) asms |
19732 | 999 |
|> ProofContext.add_assms_i LocalDefs.def_export (map #2 asms); |
27681 | 1000 |
in ([], (ctxt', Assumed axs)) end |
1001 |
| activate_elem _ _ (Defines defs) (ctxt, Derived ths) = |
|
1002 |
([], (ctxt, Derived ths)) |
|
1003 |
| activate_elem _ is_ext (Notes (kind, facts)) (ctxt, mode) = |
|
15596 | 1004 |
let |
18728 | 1005 |
val facts' = Attrib.map_facts (Attrib.attribute_i (ProofContext.theory_of ctxt)) facts; |
21441 | 1006 |
val (res, ctxt') = ctxt |> ProofContext.note_thmss_i kind facts'; |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1007 |
in (if is_ext then (map (#1 o #1) facts' ~~ map #2 res) else [], (ctxt', mode)) end; |
12502 | 1008 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1009 |
fun activate_elems ax_in_ctxt (((name, ps), mode), elems) ctxt = |
17033 | 1010 |
let |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
1011 |
val thy = ProofContext.theory_of ctxt; |
27681 | 1012 |
val (res, (ctxt', _)) = fold_map (activate_elem ax_in_ctxt (name = "")) |
1013 |
elems (ProofContext.qualified_names ctxt, mode) |
|
21441 | 1014 |
handle ERROR msg => err_in_locale ctxt msg [(name, map fst ps)]; |
15696 | 1015 |
val ctxt'' = if name = "" then ctxt' |
1016 |
else let |
|
1017 |
val ps' = map (fn (n, SOME T) => Free (n, T)) ps; |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1018 |
in if test_local_registration ctxt' (name, ps') then ctxt' |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1019 |
else let |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1020 |
val ctxt'' = put_local_registration (name, ps') ((true, ""), "") |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1021 |
(Morphism.identity, ((Vartab.empty, []), (Vartab.empty, []) )) ctxt' |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1022 |
in case mode of |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1023 |
Assumed axs => |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1024 |
fold (add_local_witness (name, ps') o |
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1025 |
Element.assume_witness thy o Element.witness_prop) axs ctxt'' |
25669 | 1026 |
| Derived ths => |
1027 |
fold (add_local_witness (name, ps')) ths ctxt'' |
|
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
1028 |
end |
15696 | 1029 |
end |
16144 | 1030 |
in (ProofContext.restore_naming ctxt ctxt'', res) end; |
13399
c136276dc847
support locale ``views'' (for cumulative predicates);
wenzelm
parents:
13394
diff
changeset
|
1031 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1032 |
fun activate_elemss ax_in_ctxt prep_facts = |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1033 |
fold_map (fn (((name, ps), mode), raw_elems) => fn ctxt => |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1034 |
let |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1035 |
val elems = map (prep_facts ctxt) raw_elems; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1036 |
val (ctxt', res) = apsnd flat |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1037 |
(activate_elems ax_in_ctxt (((name, ps), mode), elems) ctxt); |
21530 | 1038 |
val elems' = elems |> map (Element.map_ctxt_attrib Args.closure); |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1039 |
in (((((name, ps), mode), elems'), res), ctxt') end); |
12834
e5bec3268932
added locale_facts(_i) interface (useful for simple ML proof tools);
wenzelm
parents:
12806
diff
changeset
|
1040 |
|
12546 | 1041 |
in |
1042 |
||
27681 | 1043 |
(* CB: activate_facts prep_facts elemss ctxt, |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1044 |
where elemss is a list of pairs consisting of identifiers and |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1045 |
context elements, extends ctxt by the context elements yielding |
27681 | 1046 |
ctxt' and returns ((elemss', facts), ctxt'). |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1047 |
Identifiers in the argument are of the form ((name, ps), axs) and |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1048 |
assumptions use the axioms in the identifiers to set up exporters |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1049 |
in ctxt'. elemss' does not contain identifiers and is obtained |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1050 |
from elemss and the intermediate context with prep_facts. |
15703 | 1051 |
If read_facts or cert_facts is used for prep_facts, these also remove |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1052 |
the internal/external markers from elemss. *) |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1053 |
|
27681 | 1054 |
fun activate_facts ax_in_ctxt prep_facts args = |
1055 |
activate_elemss ax_in_ctxt prep_facts args |
|
1056 |
#>> (apsnd flat o split_list); |
|
15703 | 1057 |
|
12510 | 1058 |
end; |
1059 |
||
12307 | 1060 |
|
15696 | 1061 |
|
18137 | 1062 |
(** prepare locale elements **) |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1063 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1064 |
(* expressions *) |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1065 |
|
16458 | 1066 |
fun intern_expr thy (Locale xname) = Locale (intern thy xname) |
1067 |
| intern_expr thy (Merge exprs) = Merge (map (intern_expr thy) exprs) |
|
1068 |
| intern_expr thy (Rename (expr, xs)) = Rename (intern_expr thy expr, xs); |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1069 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1070 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1071 |
(* propositions and bindings *) |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1072 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1073 |
(* flatten (ctxt, prep_expr) ((ids, syn), expr) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1074 |
normalises expr (which is either a locale |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1075 |
expression or a single context element) wrt. |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1076 |
to the list ids of already accumulated identifiers. |
19783 | 1077 |
It returns ((ids', syn'), elemss) where ids' is an extension of ids |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1078 |
with identifiers generated for expr, and elemss is the list of |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1079 |
context elements generated from expr. |
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1080 |
syn and syn' are symtabs mapping parameter names to their syntax. syn' |
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1081 |
is an extension of syn. |
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1082 |
For details, see flatten_expr. |
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1083 |
|
15596 | 1084 |
Additionally, for a locale expression, the elems are grouped into a single |
1085 |
Int; individual context elements are marked Ext. In this case, the |
|
1086 |
identifier-like information of the element is as follows: |
|
1087 |
- for Fixes: (("", ps), []) where the ps have type info NONE |
|
1088 |
- for other elements: (("", []), []). |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1089 |
The implementation of activate_facts relies on identifier names being |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1090 |
empty strings for external elements. |
15596 | 1091 |
*) |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1092 |
|
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1093 |
fun flatten (ctxt, _) ((ids, syn), Elem (Fixes fixes)) = let |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1094 |
val ids' = ids @ [(("", map (Name.name_of o #1) fixes), ([], Assumed []))] |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1095 |
in |
18137 | 1096 |
((ids', |
1097 |
merge_syntax ctxt ids' |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1098 |
(syn, Symtab.make (map (fn fx => (Name.name_of (#1 fx), #3 fx)) fixes)) |
23655
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm
parents:
23591
diff
changeset
|
1099 |
handle Symtab.DUP x => err_in_locale ctxt |
d2d1138e0ddc
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
wenzelm
parents:
23591
diff
changeset
|
1100 |
("Conflicting syntax for parameter: " ^ quote x) |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1101 |
(map #1 ids')), |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1102 |
[((("", map (rpair NONE o Name.name_of o #1) fixes), Assumed []), Ext (Fixes fixes))]) |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1103 |
end |
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1104 |
| flatten _ ((ids, syn), Elem elem) = |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1105 |
((ids @ [(("", []), ([], Assumed []))], syn), [((("", []), Assumed []), Ext elem)]) |
16102
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1106 |
| flatten (ctxt, prep_expr) ((ids, syn), Expr expr) = |
c5f6726d9bb1
Locale expressions: rename with optional mixfix syntax.
ballarin
parents:
16028
diff
changeset
|
1107 |
apsnd (map (apsnd Int)) (flatten_expr ctxt ((ids, syn), prep_expr expr)); |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1108 |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1109 |
local |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1110 |
|
12839 | 1111 |
local |
1112 |
||
27681 | 1113 |
fun declare_int_elem (Fixes fixes) ctxt = |
1114 |
([], ctxt |> ProofContext.add_fixes_i (map (fn (x, T, mx) => |
|
1115 |
(x, Option.map (Term.map_type_tfree (TypeInfer.param 0)) T, mx)) fixes) |> snd) |
|
1116 |
| declare_int_elem _ ctxt = ([], ctxt); |
|
1117 |
||
1118 |
fun declare_ext_elem prep_vars (Fixes fixes) ctxt = |
|
18671 | 1119 |
let val (vars, _) = prep_vars fixes ctxt |
27681 | 1120 |
in ([], ctxt |> ProofContext.add_fixes_i vars |> snd) end |
1121 |
| declare_ext_elem prep_vars (Constrains csts) ctxt = |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1122 |
let val (_, ctxt') = prep_vars (map (fn (x, T) => (Name.binding x, SOME T, NoSyn)) csts) ctxt |
27681 | 1123 |
in ([], ctxt') end |
1124 |
| declare_ext_elem _ (Assumes asms) ctxt = (map #2 asms, ctxt) |
|
1125 |
| declare_ext_elem _ (Defines defs) ctxt = (map (fn (_, (t, ps)) => [(t, ps)]) defs, ctxt) |
|
1126 |
| declare_ext_elem _ (Notes _) ctxt = ([], ctxt); |
|
1127 |
||
1128 |
fun declare_elems prep_vars (((name, ps), Assumed _), elems) ctxt = ((case elems |
|
1129 |
of Int es => fold_map declare_int_elem es ctxt |
|
1130 |
| Ext e => declare_ext_elem prep_vars e ctxt |>> single) |
|
1131 |
handle ERROR msg => err_in_locale ctxt msg [(name, map fst ps)]) |
|
1132 |
| declare_elems _ ((_, Derived _), elems) ctxt = ([], ctxt); |
|
12727 | 1133 |
|
12839 | 1134 |
in |
1135 |
||
18671 | 1136 |
fun declare_elemss prep_vars fixed_params raw_elemss ctxt = |
12727 | 1137 |
let |
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
1138 |
(* CB: fix of type bug of goal in target with context elements. |
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
1139 |
Parameters new in context elements must receive types that are |
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
1140 |
distinct from types of parameters in target (fixed_params). *) |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1141 |
val ctxt_with_fixed = |
19900
21a99d88d925
ProofContext: moved variable operations to struct Variable;
wenzelm
parents:
19873
diff
changeset
|
1142 |
fold Variable.declare_term (map Free fixed_params) ctxt; |
12727 | 1143 |
val int_elemss = |
1144 |
raw_elemss |
|
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1145 |
|> map_filter (fn (id, Int es) => SOME (id, es) | _ => NONE) |
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
1146 |
|> unify_elemss ctxt_with_fixed fixed_params; |
27681 | 1147 |
val (raw_elemss', _) = |
1148 |
fold_map (curry (fn ((id, Int _), (_, es) :: elemss) => ((id, Int es), elemss) | x => x)) |
|
1149 |
raw_elemss int_elemss; |
|
1150 |
in fold_map (declare_elems prep_vars) raw_elemss' ctxt end; |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1151 |
|
12839 | 1152 |
end; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1153 |
|
12839 | 1154 |
local |
1155 |
||
1156 |
val norm_term = Envir.beta_norm oo Term.subst_atomic; |
|
1157 |
||
16458 | 1158 |
fun abstract_thm thy eq = |
1159 |
Thm.assume (Thm.cterm_of thy eq) |> Drule.gen_all |> Drule.abs_def; |
|
12502 | 1160 |
|
18190 | 1161 |
fun bind_def ctxt (name, ps) eq (xs, env, ths) = |
12839 | 1162 |
let |
18831 | 1163 |
val ((y, T), b) = LocalDefs.abs_def eq; |
13308 | 1164 |
val b' = norm_term env b; |
16458 | 1165 |
val th = abstract_thm (ProofContext.theory_of ctxt) eq; |
13308 | 1166 |
fun err msg = err_in_locale ctxt (msg ^ ": " ^ quote y) [(name, map fst ps)]; |
12839 | 1167 |
in |
21962 | 1168 |
exists (equal y o #1) xs andalso |
1169 |
err "Attempt to define previously specified variable"; |
|
1170 |
exists (fn (Free (y', _), _) => y = y' | _ => false) env andalso |
|
1171 |
err "Attempt to redefine variable"; |
|
16861 | 1172 |
(Term.add_frees b' xs, (Free (y, T), b') :: env, th :: ths) |
12839 | 1173 |
end; |
12575 | 1174 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1175 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1176 |
(* CB: for finish_elems (Int and Ext), |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1177 |
extracts specification, only of assumed elements *) |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1178 |
|
18190 | 1179 |
fun eval_text _ _ _ (Fixes _) text = text |
1180 |
| eval_text _ _ _ (Constrains _) text = text |
|
1181 |
| eval_text _ (_, Assumed _) is_ext (Assumes asms) |
|
1182 |
(((exts, exts'), (ints, ints')), (xs, env, defs)) = |
|
13394 | 1183 |
let |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1184 |
val ts = maps (map #1 o #2) asms; |
13394 | 1185 |
val ts' = map (norm_term env) ts; |
1186 |
val spec' = |
|
1187 |
if is_ext then ((exts @ ts, exts' @ ts'), (ints, ints')) |
|
1188 |
else ((exts, exts'), (ints @ ts, ints' @ ts')); |
|
16861 | 1189 |
in (spec', (fold Term.add_frees ts' xs, env, defs)) end |
18190 | 1190 |
| eval_text _ (_, Derived _) _ (Assumes _) text = text |
1191 |
| eval_text ctxt (id, Assumed _) _ (Defines defs) (spec, binds) = |
|
1192 |
(spec, fold (bind_def ctxt id o #1 o #2) defs binds) |
|
1193 |
| eval_text _ (_, Derived _) _ (Defines _) text = text |
|
1194 |
| eval_text _ _ _ (Notes _) text = text; |
|
13308 | 1195 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1196 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1197 |
(* for finish_elems (Int), |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1198 |
remove redundant elements of derived identifiers, |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1199 |
turn assumptions and definitions into facts, |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1200 |
satisfy hypotheses of facts *) |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1201 |
|
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1202 |
fun finish_derived _ _ (Assumed _) (Fixes fixes) = SOME (Fixes fixes) |
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1203 |
| finish_derived _ _ (Assumed _) (Constrains csts) = SOME (Constrains csts) |
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1204 |
| finish_derived _ _ (Assumed _) (Assumes asms) = SOME (Assumes asms) |
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1205 |
| finish_derived _ _ (Assumed _) (Defines defs) = SOME (Defines defs) |
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1206 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1207 |
| finish_derived _ _ (Derived _) (Fixes _) = NONE |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1208 |
| finish_derived _ _ (Derived _) (Constrains _) = NONE |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1209 |
| finish_derived sign satisfy (Derived _) (Assumes asms) = asms |
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1210 |
|> map (apsnd (map (fn (a, _) => ([Thm.assume (cterm_of sign a)], [])))) |
21441 | 1211 |
|> pair Thm.assumptionK |> Notes |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1212 |
|> Element.morph_ctxt satisfy |> SOME |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1213 |
| finish_derived sign satisfy (Derived _) (Defines defs) = defs |
17096
8327b71282ce
Improved generation of witnesses in interpretation.
ballarin
parents:
17033
diff
changeset
|
1214 |
|> map (apsnd (fn (d, _) => [([Thm.assume (cterm_of sign d)], [])])) |
21441 | 1215 |
|> pair Thm.definitionK |> Notes |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1216 |
|> Element.morph_ctxt satisfy |> SOME |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1217 |
|
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1218 |
| finish_derived _ satisfy _ (Notes facts) = Notes facts |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1219 |
|> Element.morph_ctxt satisfy |> SOME; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1220 |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1221 |
(* CB: for finish_elems (Ext) *) |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1222 |
|
13308 | 1223 |
fun closeup _ false elem = elem |
1224 |
| closeup ctxt true elem = |
|
12839 | 1225 |
let |
13308 | 1226 |
fun close_frees t = |
26206 | 1227 |
let |
1228 |
val rev_frees = |
|
1229 |
Term.fold_aterms (fn Free (x, T) => |
|
1230 |
if Variable.is_fixed ctxt x then I else insert (op =) (x, T) | _ => I) t []; |
|
26299
2f387f5c0f52
closeup: recover original order of free variables!
wenzelm
parents:
26206
diff
changeset
|
1231 |
in Term.list_all_free (rev rev_frees, t) end; |
13308 | 1232 |
|
1233 |
fun no_binds [] = [] |
|
18678 | 1234 |
| no_binds _ = error "Illegal term bindings in locale element"; |
13308 | 1235 |
in |
1236 |
(case elem of |
|
1237 |
Assumes asms => Assumes (asms |> map (fn (a, propps) => |
|
19585 | 1238 |
(a, map (fn (t, ps) => (close_frees t, no_binds ps)) propps))) |
13308 | 1239 |
| Defines defs => Defines (defs |> map (fn (a, (t, ps)) => |
18831 | 1240 |
(a, (close_frees (#2 (LocalDefs.cert_def ctxt t)), no_binds ps)))) |
13308 | 1241 |
| e => e) |
1242 |
end; |
|
12839 | 1243 |
|
12502 | 1244 |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1245 |
fun finish_ext_elem parms _ (Fixes fixes, _) = Fixes (map (fn (binding, _, mx) => |
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1246 |
let val x = Name.name_of binding |
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1247 |
in (binding, AList.lookup (op =) parms x, mx) end) fixes) |
18899
a8e913c93578
theorem(_in_locale): Element.statement, Obtain.statement;
wenzelm
parents:
18890
diff
changeset
|
1248 |
| finish_ext_elem parms _ (Constrains _, _) = Constrains [] |
12839 | 1249 |
| finish_ext_elem _ close (Assumes asms, propp) = |
1250 |
close (Assumes (map #1 asms ~~ propp)) |
|
1251 |
| finish_ext_elem _ close (Defines defs, propp) = |
|
19585 | 1252 |
close (Defines (map #1 defs ~~ map (fn [(t, ps)] => (t, ps)) propp)) |
12839 | 1253 |
| finish_ext_elem _ _ (Notes facts, _) = Notes facts; |
1254 |
||
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1255 |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1256 |
(* CB: finish_parms introduces type info from parms to identifiers *) |
15531 | 1257 |
(* CB: only needed for types that have been NONE so far??? |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1258 |
If so, which are these??? *) |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1259 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1260 |
fun finish_parms parms (((name, ps), mode), elems) = |
19932 | 1261 |
(((name, map (fn (x, _) => (x, AList.lookup (op = : string * string -> bool) parms x)) ps), mode), elems); |
12839 | 1262 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1263 |
fun finish_elems ctxt parms _ ((text, wits), ((id, Int e), _)) = |
12839 | 1264 |
let |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1265 |
val [(id' as (_, mode), es)] = unify_elemss ctxt parms [(id, e)]; |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1266 |
val wits' = case mode of Assumed _ => wits | Derived ths => wits @ ths; |
18190 | 1267 |
val text' = fold (eval_text ctxt id' false) es text; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1268 |
val es' = map_filter |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1269 |
(finish_derived (ProofContext.theory_of ctxt) (Element.satisfy_morphism wits') mode) es; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1270 |
in ((text', wits'), (id', map Int es')) end |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1271 |
| finish_elems ctxt parms do_close ((text, wits), ((id, Ext e), [propp])) = |
13308 | 1272 |
let |
1273 |
val e' = finish_ext_elem parms (closeup ctxt do_close) (e, propp); |
|
18190 | 1274 |
val text' = eval_text ctxt id true e' text; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1275 |
in ((text', wits), (id, [Ext e'])) end |
12839 | 1276 |
|
1277 |
in |
|
12510 | 1278 |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1279 |
(* CB: only called by prep_elemss *) |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1280 |
|
13375 | 1281 |
fun finish_elemss ctxt parms do_close = |
1282 |
foldl_map (apsnd (finish_parms parms) o finish_elems ctxt parms do_close); |
|
12839 | 1283 |
|
1284 |
end; |
|
1285 |
||
16736
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1286 |
|
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1287 |
(* Remove duplicate Defines elements: temporary workaround to fix Afp/Category. *) |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1288 |
|
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1289 |
fun defs_ord (defs1, defs2) = |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1290 |
list_ord (fn ((_, (d1, _)), (_, (d2, _))) => |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1291 |
Term.fast_term_ord (d1, d2)) (defs1, defs2); |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1292 |
structure Defstab = |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
1293 |
TableFun(type key = (Attrib.binding * (term * term list)) list val ord = defs_ord); |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1294 |
|
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1295 |
fun rem_dup_defs es ds = |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1296 |
fold_map (fn e as (Defines defs) => (fn ds => |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1297 |
if Defstab.defined ds defs |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1298 |
then (Defines [], ds) |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1299 |
else (e, Defstab.update (defs, ()) ds)) |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1300 |
| e => (fn ds => (e, ds))) es ds; |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1301 |
fun rem_dup_elemss (Int es) ds = apfst Int (rem_dup_defs es ds) |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1302 |
| rem_dup_elemss (Ext e) ds = (Ext e, ds); |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1303 |
fun rem_dup_defines raw_elemss = |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1304 |
fold_map (fn (id as (_, (Assumed _)), es) => (fn ds => |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1305 |
apfst (pair id) (rem_dup_elemss es ds)) |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1306 |
| (id as (_, (Derived _)), es) => (fn ds => |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1307 |
((id, es), ds))) raw_elemss Defstab.empty |> #1; |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1308 |
|
16736
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1309 |
(* CB: type inference and consistency checks for locales. |
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1310 |
|
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1311 |
Works by building a context (through declare_elemss), extracting the |
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1312 |
required information and adjusting the context elements (finish_elemss). |
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1313 |
Can also universally close free vars in assms and defs. This is only |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1314 |
needed for Ext elements and controlled by parameter do_close. |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1315 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1316 |
Only elements of assumed identifiers are considered. |
16736
1e792b32abef
Preparations for interpretation of locales in locales.
ballarin
parents:
16620
diff
changeset
|
1317 |
*) |
15127 | 1318 |
|
18671 | 1319 |
fun prep_elemss prep_vars prepp do_close context fixed_params raw_elemss raw_concl = |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1320 |
let |
15127 | 1321 |
(* CB: contexts computed in the course of this function are discarded. |
1322 |
They are used for type inference and consistency checks only. *) |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1323 |
(* CB: fixed_params are the parameters (with types) of the target locale, |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1324 |
empty list if there is no target. *) |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1325 |
(* CB: raw_elemss are list of pairs consisting of identifiers and |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1326 |
context elements, the latter marked as internal or external. *) |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1327 |
val raw_elemss = rem_dup_defines raw_elemss; |
27681 | 1328 |
val (raw_proppss, raw_ctxt) = declare_elemss prep_vars fixed_params raw_elemss context; |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1329 |
(* CB: raw_ctxt is context with additional fixed variables derived from |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1330 |
the fixes elements in raw_elemss, |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1331 |
raw_proppss contains assumptions and definitions from the |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1332 |
external elements in raw_elemss. *) |
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1333 |
fun prep_prop raw_propp (raw_ctxt, raw_concl) = |
18450
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1334 |
let |
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1335 |
(* CB: add type information from fixed_params to context (declare_term) *) |
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1336 |
(* CB: process patterns (conclusion and external elements only) *) |
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1337 |
val (ctxt, all_propp) = |
19900
21a99d88d925
ProofContext: moved variable operations to struct Variable;
wenzelm
parents:
19873
diff
changeset
|
1338 |
prepp (fold Variable.declare_term (map Free fixed_params) raw_ctxt, raw_concl @ raw_propp); |
18450
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1339 |
(* CB: add type information from conclusion and external elements to context *) |
19900
21a99d88d925
ProofContext: moved variable operations to struct Variable;
wenzelm
parents:
19873
diff
changeset
|
1340 |
val ctxt = fold Variable.declare_term (maps (map fst) all_propp) ctxt; |
18450
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1341 |
(* CB: resolve schematic variables (patterns) in conclusion and external elements. *) |
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1342 |
val all_propp' = map2 (curry (op ~~)) |
e57731ba01dd
discontinued unflat in favour of burrow and burrow_split
haftmann
parents:
18421
diff
changeset
|
1343 |
(#1 (#2 (ProofContext.bind_propp_schematic_i (ctxt, all_propp)))) (map (map snd) all_propp); |
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
1344 |
val (concl, propp) = chop (length raw_concl) all_propp'; |
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1345 |
in (propp, (ctxt, concl)) end |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1346 |
|
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1347 |
val (proppss, (ctxt, concl)) = |
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1348 |
(fold_burrow o fold_burrow) prep_prop raw_proppss (raw_ctxt, raw_concl); |
12502 | 1349 |
|
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1350 |
(* CB: obtain all parameters from identifier part of raw_elemss *) |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1351 |
val xs = map #1 (params_of' raw_elemss); |
12727 | 1352 |
val typing = unify_frozen ctxt 0 |
19900
21a99d88d925
ProofContext: moved variable operations to struct Variable;
wenzelm
parents:
19873
diff
changeset
|
1353 |
(map (Variable.default_type raw_ctxt) xs) |
21a99d88d925
ProofContext: moved variable operations to struct Variable;
wenzelm
parents:
19873
diff
changeset
|
1354 |
(map (Variable.default_type ctxt) xs); |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1355 |
val parms = param_types (xs ~~ typing); |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1356 |
(* CB: parms are the parameters from raw_elemss, with correct typing. *) |
12273 | 1357 |
|
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1358 |
(* CB: extract information from assumes and defines elements |
16169
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
1359 |
(fixes, constrains and notes in raw_elemss don't have an effect on |
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
1360 |
text and elemss), compute final form of context elements. *) |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1361 |
val ((text, _), elemss) = finish_elemss ctxt parms do_close |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1362 |
((((([], []), ([], [])), ([], [], [])), []), raw_elemss ~~ proppss); |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1363 |
(* CB: text has the following structure: |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1364 |
(((exts, exts'), (ints, ints')), (xs, env, defs)) |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1365 |
where |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1366 |
exts: external assumptions (terms in external assumes elements) |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1367 |
exts': dito, normalised wrt. env |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1368 |
ints: internal assumptions (terms in internal assumes elements) |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1369 |
ints': dito, normalised wrt. env |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1370 |
xs: the free variables in exts' and ints' and rhss of definitions, |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1371 |
this includes parameters except defined parameters |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1372 |
env: list of term pairs encoding substitutions, where the first term |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1373 |
is a free variable; substitutions represent defines elements and |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1374 |
the rhs is normalised wrt. the previous env |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1375 |
defs: theorems representing the substitutions from defines elements |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1376 |
(thms are normalised wrt. env). |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1377 |
elemss is an updated version of raw_elemss: |
16169
b59202511b8a
Locales: new element constrains, parameter renaming with syntax,
ballarin
parents:
16144
diff
changeset
|
1378 |
- type info added to Fixes and modified in Constrains |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1379 |
- axiom and definition statement replaced by corresponding one |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1380 |
from proppss in Assumes and Defines |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1381 |
- Facts unchanged |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1382 |
*) |
13308 | 1383 |
in ((parms, elemss, concl), text) end; |
12502 | 1384 |
|
1385 |
in |
|
1386 |
||
18671 | 1387 |
fun read_elemss x = prep_elemss ProofContext.read_vars ProofContext.read_propp_schematic x; |
1388 |
fun cert_elemss x = prep_elemss ProofContext.cert_vars ProofContext.cert_propp_schematic x; |
|
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1389 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1390 |
end; |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1391 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1392 |
|
15703 | 1393 |
(* facts and attributes *) |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1394 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1395 |
local |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1396 |
|
20965 | 1397 |
fun check_name name = |
18678 | 1398 |
if NameSpace.is_qualified name then error ("Illegal qualified name: " ^ quote name) |
15703 | 1399 |
else name; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1400 |
|
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
1401 |
fun prep_facts _ _ _ ctxt (Int elem) = elem |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
1402 |
|> Element.morph_ctxt (Morphism.thm_morphism (Thm.transfer (ProofContext.theory_of ctxt))) |
20965 | 1403 |
| prep_facts prep_name get intern ctxt (Ext elem) = elem |> Element.map_ctxt |
15703 | 1404 |
{var = I, typ = I, term = I, |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1405 |
name = Name.map_name prep_name, |
15703 | 1406 |
fact = get ctxt, |
16458 | 1407 |
attrib = Args.assignable o intern (ProofContext.theory_of ctxt)}; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1408 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1409 |
in |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1410 |
|
26345
f70620a4cf81
renamed former get_thms(_silent) to get_fact(_silent);
wenzelm
parents:
26299
diff
changeset
|
1411 |
fun read_facts x = prep_facts check_name ProofContext.get_fact Attrib.intern_src x; |
20965 | 1412 |
fun cert_facts x = prep_facts I (K I) (K I) x; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1413 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1414 |
end; |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1415 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1416 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1417 |
(* Get the specification of a locale *) |
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1418 |
|
19780 | 1419 |
(*The global specification is made from the parameters and global |
1420 |
assumptions, the local specification from the parameters and the |
|
1421 |
local assumptions.*) |
|
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1422 |
|
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1423 |
local |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1424 |
|
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1425 |
fun gen_asms_of get thy name = |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1426 |
let |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1427 |
val ctxt = ProofContext.init thy; |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1428 |
val (_, raw_elemss) = flatten (ctxt, I) (([], Symtab.empty), Expr (Locale name)); |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1429 |
val ((_, elemss, _), _) = read_elemss false ctxt [] raw_elemss []; |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1430 |
in |
18890 | 1431 |
elemss |> get |
19780 | 1432 |
|> maps (fn (_, es) => map (fn Int e => e) es) |
1433 |
|> maps (fn Assumes asms => asms | _ => []) |
|
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1434 |
|> map (apsnd (map fst)) |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1435 |
end; |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1436 |
|
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1437 |
in |
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1438 |
|
25619 | 1439 |
fun parameters_of thy = #params o the_locale thy; |
1440 |
||
1441 |
fun intros thy = #intros o the_locale thy; |
|
1442 |
(*returns introduction rule for delta predicate and locale predicate |
|
1443 |
as a pair of singleton lists*) |
|
1444 |
||
1445 |
fun dests thy = #dests o the_locale thy; |
|
1446 |
||
27709 | 1447 |
fun facts_of thy = map_filter (fn (Element.Notes (_, facts), _) => SOME facts |
1448 |
| _ => NONE) o #elems o the_locale thy; |
|
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1449 |
|
19276 | 1450 |
fun parameters_of_expr thy expr = |
1451 |
let |
|
1452 |
val ctxt = ProofContext.init thy; |
|
19783 | 1453 |
val pts = params_of_expr ctxt [] (intern_expr thy expr) |
1454 |
([], Symtab.empty, Symtab.empty); |
|
1455 |
val raw_params_elemss = make_raw_params_elemss pts; |
|
19276 | 1456 |
val ((_, syn), raw_elemss) = flatten (ctxt, intern_expr thy) |
1457 |
(([], Symtab.empty), Expr expr); |
|
19783 | 1458 |
val ((parms, _, _), _) = |
1459 |
read_elemss false ctxt [] (raw_params_elemss @ raw_elemss) []; |
|
19276 | 1460 |
in map (fn p as (n, _) => (p, Symtab.lookup syn n |> the)) parms end; |
1461 |
||
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1462 |
fun local_asms_of thy name = |
18890 | 1463 |
gen_asms_of (single o Library.last_elem) thy name; |
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1464 |
|
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1465 |
fun global_asms_of thy name = |
18890 | 1466 |
gen_asms_of I thy name; |
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1467 |
|
19780 | 1468 |
end; |
18795
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1469 |
|
303793f49b0f
Interface to access the specification of a named locale.
ballarin
parents:
18782
diff
changeset
|
1470 |
|
22573 | 1471 |
(* full context statements: imports + elements + conclusion *) |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1472 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1473 |
local |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1474 |
|
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1475 |
fun prep_context_statement prep_expr prep_elemss prep_facts |
22573 | 1476 |
do_close fixed_params imports elements raw_concl context = |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1477 |
let |
16458 | 1478 |
val thy = ProofContext.theory_of context; |
13375 | 1479 |
|
19783 | 1480 |
val (import_params, import_tenv, import_syn) = |
22573 | 1481 |
params_of_expr context fixed_params (prep_expr thy imports) |
19783 | 1482 |
([], Symtab.empty, Symtab.empty); |
1483 |
val includes = map_filter (fn Expr e => SOME e | Elem _ => NONE) elements; |
|
1484 |
val (incl_params, incl_tenv, incl_syn) = fold (params_of_expr context fixed_params) |
|
1485 |
(map (prep_expr thy) includes) (import_params, import_tenv, import_syn); |
|
1486 |
||
1487 |
val ((import_ids, _), raw_import_elemss) = |
|
22573 | 1488 |
flatten (context, prep_expr thy) (([], Symtab.empty), Expr imports); |
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
1489 |
(* CB: normalise "includes" among elements *) |
16458 | 1490 |
val ((ids, syn), raw_elemsss) = foldl_map (flatten (context, prep_expr thy)) |
19783 | 1491 |
((import_ids, incl_syn), elements); |
15696 | 1492 |
|
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1493 |
val raw_elemss = flat raw_elemsss; |
14508
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1494 |
(* CB: raw_import_elemss @ raw_elemss is the normalised list of |
859b11514537
Experimental command for instantiation of locales in proof contexts:
ballarin
parents:
14446
diff
changeset
|
1495 |
context elements obtained from import and elements. *) |
19783 | 1496 |
(* Now additional elements for parameters are inserted. *) |
1497 |
val import_params_ids = make_params_ids import_params; |
|
1498 |
val incl_params_ids = |
|
1499 |
make_params_ids (incl_params \\ import_params); |
|
1500 |
val raw_import_params_elemss = |
|
1501 |
make_raw_params_elemss (import_params, incl_tenv, incl_syn); |
|
1502 |
val raw_incl_params_elemss = |
|
1503 |
make_raw_params_elemss (incl_params \\ import_params, incl_tenv, incl_syn); |
|
13375 | 1504 |
val ((parms, all_elemss, concl), (spec, (_, _, defs))) = prep_elemss do_close |
19783 | 1505 |
context fixed_params |
1506 |
(raw_import_params_elemss @ raw_import_elemss @ raw_incl_params_elemss @ raw_elemss) raw_concl; |
|
1507 |
||
15696 | 1508 |
(* replace extended ids (for axioms) by ids *) |
19783 | 1509 |
val (import_ids', incl_ids) = chop (length import_ids) ids; |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
1510 |
val all_ids = import_params_ids @ import_ids' @ incl_params_ids @ incl_ids; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1511 |
val all_elemss' = map (fn (((_, ps), _), (((n, ps'), mode), elems)) => |
17485 | 1512 |
(((n, map (fn p => (p, (the o AList.lookup (op =) ps') p)) ps), mode), elems)) |
20035
80c79876d2de
Internal restructuring: identify no longer computes syntax.
ballarin
parents:
20032
diff
changeset
|
1513 |
(all_ids ~~ all_elemss); |
19783 | 1514 |
(* CB: all_elemss and parms contain the correct parameter types *) |
15696 | 1515 |
|
19783 | 1516 |
val (ps, qs) = chop (length raw_import_params_elemss + length raw_import_elemss) all_elemss'; |
27681 | 1517 |
val ((import_elemss, _), import_ctxt) = |
1518 |
activate_facts false prep_facts ps context; |
|
1519 |
||
1520 |
val ((elemss, _), ctxt) = |
|
1521 |
activate_facts false prep_facts qs (ProofContext.set_stmt true import_ctxt); |
|
12834
e5bec3268932
added locale_facts(_i) interface (useful for simple ML proof tools);
wenzelm
parents:
12806
diff
changeset
|
1522 |
in |
19783 | 1523 |
((((import_ctxt, import_elemss), (ctxt, elemss, syn)), |
19991
0c9650664d47
Locales no longer generate views. The following functions have changed
ballarin
parents:
19984
diff
changeset
|
1524 |
(parms, spec, defs)), concl) |
12834
e5bec3268932
added locale_facts(_i) interface (useful for simple ML proof tools);
wenzelm
parents:
12806
diff
changeset
|
1525 |
end; |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1526 |
|
18806 | 1527 |
fun prep_statement prep_locale prep_ctxt raw_locale elems concl ctxt = |
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1528 |
let |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1529 |
val thy = ProofContext.theory_of ctxt; |
16458 | 1530 |
val locale = Option.map (prep_locale thy) raw_locale; |
22573 | 1531 |
val (fixed_params, imports) = |
18806 | 1532 |
(case locale of |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1533 |
NONE => ([], empty) |
15531 | 1534 |
| SOME name => |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1535 |
let val {params = ps, ...} = the_locale thy name |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1536 |
in (map fst ps, Locale name) end); |
19991
0c9650664d47
Locales no longer generate views. The following functions have changed
ballarin
parents:
19984
diff
changeset
|
1537 |
val ((((locale_ctxt, _), (elems_ctxt, _, _)), _), concl') = |
22573 | 1538 |
prep_ctxt false fixed_params imports elems concl ctxt; |
19991
0c9650664d47
Locales no longer generate views. The following functions have changed
ballarin
parents:
19984
diff
changeset
|
1539 |
in (locale, locale_ctxt, elems_ctxt, concl') end; |
13399
c136276dc847
support locale ``views'' (for cumulative predicates);
wenzelm
parents:
13394
diff
changeset
|
1540 |
|
22573 | 1541 |
fun prep_expr prep imports body ctxt = |
19780 | 1542 |
let |
22573 | 1543 |
val (((_, import_elemss), (ctxt', elemss, _)), _) = prep imports body ctxt; |
19780 | 1544 |
val all_elems = maps snd (import_elemss @ elemss); |
1545 |
in (all_elems, ctxt') end; |
|
1546 |
||
12529
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1547 |
in |
d99716a53f59
simultaneous type-inference of complete context/statement specifications;
wenzelm
parents:
12514
diff
changeset
|
1548 |
|
18806 | 1549 |
val read_ctxt = prep_context_statement intern_expr read_elemss read_facts; |
1550 |
val cert_ctxt = prep_context_statement (K I) cert_elemss cert_facts; |
|
14215
ebf291f3b449
Improvements to Isar/Locales: premises generated by "includes" elements
ballarin
parents:
13629
diff
changeset
|
1551 |
|
22573 | 1552 |
fun read_context imports body ctxt = #1 (read_ctxt true [] imports (map Elem body) [] ctxt); |
1553 |
fun cert_context imports body ctxt = #1 (cert_ctxt true [] imports (map Elem body) [] ctxt); |
|
12502 | 1554 |
|
19780 | 1555 |
val read_expr = prep_expr read_context; |
1556 |
val cert_expr = prep_expr cert_context; |
|
1557 |
||
21035 | 1558 |
fun read_context_statement loc = prep_statement intern read_ctxt loc; |
1559 |
fun read_context_statement_i loc = prep_statement (K I) read_ctxt loc; |
|
1560 |
fun cert_context_statement loc = prep_statement (K I) cert_ctxt loc; |
|
18806 | 1561 |
|
12502 | 1562 |
end; |
11896 | 1563 |
|
1564 |
||
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1565 |
(* init *) |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1566 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1567 |
fun init loc = |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1568 |
ProofContext.init |
25669 | 1569 |
#> #2 o cert_context_statement (SOME loc) [] []; |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1570 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1571 |
|
13336 | 1572 |
(* print locale *) |
12070 | 1573 |
|
22573 | 1574 |
fun print_locale thy show_facts imports body = |
1575 |
let val (all_elems, ctxt) = read_expr imports body (ProofContext.init thy) in |
|
18137 | 1576 |
Pretty.big_list "locale elements:" (all_elems |
17316 | 1577 |
|> (if show_facts then I else filter (fn Notes _ => false | _ => true)) |
21701 | 1578 |
|> map (Element.pretty_ctxt ctxt) |> filter_out null |
1579 |
|> map Pretty.chunks) |
|
13336 | 1580 |
|> Pretty.writeln |
12277 | 1581 |
end; |
12070 | 1582 |
|
1583 |
||
12706 | 1584 |
|
16144 | 1585 |
(** store results **) |
12702 | 1586 |
|
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
1587 |
(* naming of interpreted theorems *) |
15696 | 1588 |
|
28107 | 1589 |
fun add_param_prefixss s = (map o apfst o apfst) (Name.qualified s); |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1590 |
fun drop_param_prefixss args = (map o apfst o apfst o Name.map_name) |
28053 | 1591 |
(fn "" => "" | s => (NameSpace.implode o tl o NameSpace.explode) s) args; |
1592 |
||
1593 |
fun global_note_prefix_i kind loc (fully_qualified, prfx) args thy = |
|
16144 | 1594 |
thy |
22796 | 1595 |
|> Sign.qualified_names |
26645
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
1596 |
|> Sign.add_path (NameSpace.base loc ^ "_locale") |
22796 | 1597 |
|> (if fully_qualified then Sign.sticky_prefix prfx else Sign.add_path prfx) |
28053 | 1598 |
|> PureThy.note_thmss kind (if fully_qualified then args else drop_param_prefixss args) |
22796 | 1599 |
||> Sign.restore_naming thy; |
15696 | 1600 |
|
28053 | 1601 |
fun local_note_prefix_i kind loc (fully_qualified, prfx) args ctxt = |
16144 | 1602 |
ctxt |
19061
ffbbac0261c9
removed distinct, renamed gen_distinct to distinct;
wenzelm
parents:
19025
diff
changeset
|
1603 |
|> ProofContext.qualified_names |
26645
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
1604 |
|> ProofContext.add_path (NameSpace.base loc ^ "_locale") |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1605 |
|> (if fully_qualified then ProofContext.sticky_prefix prfx else ProofContext.add_path prfx) |
28053 | 1606 |
|> ProofContext.note_thmss_i kind (if fully_qualified then args else drop_param_prefixss args) |
19780 | 1607 |
||> ProofContext.restore_naming ctxt; |
16144 | 1608 |
|
15696 | 1609 |
|
23918 | 1610 |
(* join equations of an id with already accumulated ones *) |
1611 |
||
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1612 |
fun join_eqns get_reg id eqns = |
23918 | 1613 |
let |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1614 |
val eqns' = case get_reg id |
23918 | 1615 |
of NONE => eqns |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1616 |
| SOME (_, _, eqns') => Termtab.join (fn _ => fn (_, e) => e) (eqns, eqns') |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1617 |
(* prefer equations from eqns' *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1618 |
in ((id, eqns'), eqns') end; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1619 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1620 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1621 |
(* collect witnesses and equations up to a particular target for a |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
1622 |
registration; requires parameters and flattened list of identifiers |
17138 | 1623 |
instead of recomputing it from the target *) |
1624 |
||
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1625 |
fun collect_witnesses ctxt (imprt as ((impT, _), (imp, _))) parms ids ext_ts = let |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1626 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1627 |
val thy = ProofContext.theory_of ctxt; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1628 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1629 |
val ts = map (var_inst_term (impT, imp)) ext_ts; |
17138 | 1630 |
val (parms, parmTs) = split_list parms; |
19810 | 1631 |
val parmvTs = map Logic.varifyT parmTs; |
17138 | 1632 |
val vtinst = fold (Sign.typ_match thy) (parmvTs ~~ map Term.fastype_of ts) Vartab.empty; |
1633 |
val tinst = Vartab.dest vtinst |> map (fn ((x, 0), (_, T)) => (x, T)) |
|
18137 | 1634 |
|> Symtab.make; |
17138 | 1635 |
val inst = Symtab.make (parms ~~ ts); |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1636 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1637 |
(* instantiate parameter names in ids *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1638 |
val ext_inst = Symtab.make (parms ~~ ext_ts); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1639 |
fun ext_inst_names ps = map (the o Symtab.lookup ext_inst) ps; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1640 |
val inst_ids = map (apfst (apsnd ext_inst_names)) ids; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1641 |
val assumed_ids = map_filter (fn (id, (_, Assumed _)) => SOME id | _ => NONE) inst_ids; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1642 |
val wits = maps (#2 o the o get_local_registration ctxt imprt) assumed_ids; |
23918 | 1643 |
val eqns = |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1644 |
fold_map (join_eqns (get_local_registration ctxt imprt)) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1645 |
(map fst inst_ids) Termtab.empty |> snd |> Termtab.dest |> map snd; |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1646 |
in ((tinst, inst), wits, eqns) end; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1647 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1648 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1649 |
(* standardise export morphism *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1650 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1651 |
(* clone from Element.generalize_facts *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1652 |
fun standardize thy export facts = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1653 |
let |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1654 |
val exp_fact = Drule.zero_var_indexes_list o map Thm.strip_shyps o Morphism.fact export; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1655 |
val exp_term = TermSubst.zero_var_indexes o Morphism.term export; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1656 |
(* FIXME sync with exp_fact *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1657 |
val exp_typ = Logic.type_map exp_term; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1658 |
val morphism = |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1659 |
Morphism.morphism {name = I, var = I, typ = exp_typ, term = exp_term, fact = exp_fact}; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1660 |
in Element.facts_map (Element.morph_ctxt morphism) facts end; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1661 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1662 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1663 |
fun morph_ctxt' phi = Element.map_ctxt |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1664 |
{name = I, |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1665 |
var = Morphism.var phi, |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1666 |
typ = Morphism.typ phi, |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1667 |
term = Morphism.term phi, |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1668 |
fact = Morphism.fact phi, |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1669 |
attrib = Args.morph_values phi}; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1670 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1671 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1672 |
(* compute morphism and apply to args *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
1673 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1674 |
fun inst_morph thy prfx param_prfx insts prems eqns = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1675 |
Morphism.name_morphism (Name.qualified prfx o Name.qualified param_prfx) $> |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1676 |
Element.inst_morphism thy insts $> Element.satisfy_morphism prems $> |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1677 |
Morphism.term_morphism (MetaSimplifier.rewrite_term thy eqns []) $> |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1678 |
Morphism.thm_morphism (MetaSimplifier.rewrite_rule eqns); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1679 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1680 |
fun interpret_args thy inst exp attrib args = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1681 |
args |> Element.facts_map (morph_ctxt' inst) |> |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1682 |
(* morph_ctxt' suppresses application of name morphism. FIXME *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1683 |
standardize thy exp |> Attrib.map_facts attrib; |
17138 | 1684 |
|
1685 |
||
15696 | 1686 |
(* store instantiations of args for all registered interpretations |
1687 |
of the theory *) |
|
1688 |
||
21441 | 1689 |
fun note_thmss_registrations target (kind, args) thy = |
15596 | 1690 |
let |
19278 | 1691 |
val parms = the_locale thy target |> #params |> map fst; |
16458 | 1692 |
val ids = flatten (ProofContext.init thy, intern_expr thy) |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
1693 |
(([], Symtab.empty), Expr (Locale target)) |> fst |> fst; |
15696 | 1694 |
|
1695 |
val regs = get_global_registrations thy target; |
|
1696 |
(* add args to thy for all registrations *) |
|
15596 | 1697 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1698 |
fun activate (ext_ts, (((fully_qualified, prfx), pprfx), (exp, imp), _, _)) thy = |
15696 | 1699 |
let |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1700 |
val (insts, prems, eqns) = collect_witnesses (ProofContext.init thy) imp parms ids ext_ts; |
20911 | 1701 |
val attrib = Attrib.attribute_i thy; |
28053 | 1702 |
val args' = args |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1703 |
|> interpret_args thy (inst_morph thy prfx pprfx insts prems eqns) exp attrib |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
1704 |
|> add_param_prefixss pprfx; |
28053 | 1705 |
in global_note_prefix_i kind target (fully_qualified, prfx) args' thy |> snd end; |
18190 | 1706 |
in fold activate regs thy end; |
15596 | 1707 |
|
1708 |
||
20911 | 1709 |
(* locale results *) |
12958 | 1710 |
|
21441 | 1711 |
fun add_thmss loc kind args ctxt = |
12706 | 1712 |
let |
27681 | 1713 |
val (([(_, [Notes args'])], _), ctxt') = |
21441 | 1714 |
activate_facts true cert_facts |
27681 | 1715 |
[((("", []), Assumed []), [Ext (Notes (kind, args))])] ctxt; |
20911 | 1716 |
val ctxt'' = ctxt' |> ProofContext.theory |
1717 |
(change_locale loc |
|
27716 | 1718 |
(fn (axiom, elems, params, decls, regs, intros, dests) => |
1719 |
(axiom, elems @ [(Notes args', stamp ())], |
|
1720 |
params, decls, regs, intros, dests)) |
|
21441 | 1721 |
#> note_thmss_registrations loc args'); |
21582 | 1722 |
in ctxt'' end; |
15703 | 1723 |
|
11896 | 1724 |
|
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1725 |
(* declarations *) |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1726 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1727 |
local |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1728 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1729 |
fun decl_attrib decl phi = Thm.declaration_attribute (K (decl phi)); |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1730 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1731 |
fun add_decls add loc decl = |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1732 |
ProofContext.theory (change_locale loc |
27716 | 1733 |
(fn (axiom, elems, params, decls, regs, intros, dests) => |
1734 |
(axiom, elems, params, add (decl, stamp ()) decls, regs, intros, dests))) #> |
|
24006 | 1735 |
add_thmss loc Thm.internalK |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1736 |
[((Name.no_binding, [Attrib.internal (decl_attrib decl)]), [([Drule.dummy_thm], [])])]; |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1737 |
|
23418 | 1738 |
in |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1739 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1740 |
val add_type_syntax = add_decls (apfst o cons); |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1741 |
val add_term_syntax = add_decls (apsnd o cons); |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1742 |
val add_declaration = add_decls (K I); |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1743 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1744 |
end; |
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1745 |
|
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1746 |
|
18137 | 1747 |
|
1748 |
(** define locales **) |
|
1749 |
||
13336 | 1750 |
(* predicate text *) |
15596 | 1751 |
(* CB: generate locale predicates and delta predicates *) |
13336 | 1752 |
|
13375 | 1753 |
local |
1754 |
||
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1755 |
(* introN: name of theorems for introduction rules of locale and |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1756 |
delta predicates; |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1757 |
axiomsN: name of theorem set with destruct rules for locale predicates, |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1758 |
also name suffix of delta predicates. *) |
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1759 |
|
13375 | 1760 |
val introN = "intro"; |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1761 |
val axiomsN = "axioms"; |
13375 | 1762 |
|
16458 | 1763 |
fun atomize_spec thy ts = |
13375 | 1764 |
let |
23418 | 1765 |
val t = Logic.mk_conjunction_balanced ts; |
16458 | 1766 |
val body = ObjectLogic.atomize_term thy t; |
13375 | 1767 |
val bodyT = Term.fastype_of body; |
1768 |
in |
|
16458 | 1769 |
if bodyT = propT then (t, propT, Thm.reflexive (Thm.cterm_of thy t)) |
23591 | 1770 |
else (body, bodyT, ObjectLogic.atomize (Thm.cterm_of thy t)) |
13375 | 1771 |
end; |
1772 |
||
25073
13db30d367d2
locale pred: authentic syntax, tuned aprop_tr' accordingly;
wenzelm
parents:
25067
diff
changeset
|
1773 |
fun aprop_tr' n c = (Syntax.constN ^ c, fn ctxt => fn args => |
13db30d367d2
locale pred: authentic syntax, tuned aprop_tr' accordingly;
wenzelm
parents:
25067
diff
changeset
|
1774 |
if length args = n then |
13db30d367d2
locale pred: authentic syntax, tuned aprop_tr' accordingly;
wenzelm
parents:
25067
diff
changeset
|
1775 |
Syntax.const "_aprop" $ |
13db30d367d2
locale pred: authentic syntax, tuned aprop_tr' accordingly;
wenzelm
parents:
25067
diff
changeset
|
1776 |
Term.list_comb (Syntax.free (Consts.extern (ProofContext.consts_of ctxt) c), args) |
13394 | 1777 |
else raise Match); |
13336 | 1778 |
|
15104 | 1779 |
(* CB: define one predicate including its intro rule and axioms |
1780 |
- bname: predicate name |
|
1781 |
- parms: locale parameters |
|
1782 |
- defs: thms representing substitutions from defines elements |
|
1783 |
- ts: terms representing locale assumptions (not normalised wrt. defs) |
|
1784 |
- norm_ts: terms representing locale assumptions (normalised wrt. defs) |
|
1785 |
- thy: the theory |
|
1786 |
*) |
|
1787 |
||
13420 | 1788 |
fun def_pred bname parms defs ts norm_ts thy = |
13375 | 1789 |
let |
16458 | 1790 |
val name = Sign.full_name thy bname; |
13375 | 1791 |
|
16458 | 1792 |
val (body, bodyT, body_eq) = atomize_spec thy norm_ts; |
13394 | 1793 |
val env = Term.add_term_free_names (body, []); |
20664 | 1794 |
val xs = filter (member (op =) env o #1) parms; |
13394 | 1795 |
val Ts = map #2 xs; |
23178 | 1796 |
val extraTs = (Term.term_tfrees body \\ List.foldr Term.add_typ_tfrees [] Ts) |
13394 | 1797 |
|> Library.sort_wrt #1 |> map TFree; |
13399
c136276dc847
support locale ``views'' (for cumulative predicates);
wenzelm
parents:
13394
diff
changeset
|
1798 |
val predT = map Term.itselfT extraTs ---> Ts ---> bodyT; |
13336 | 1799 |
|
13394 | 1800 |
val args = map Logic.mk_type extraTs @ map Free xs; |
1801 |
val head = Term.list_comb (Const (name, predT), args); |
|
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
1802 |
val statement = ObjectLogic.ensure_propT thy head; |
13375 | 1803 |
|
18358 | 1804 |
val ([pred_def], defs_thy) = |
13375 | 1805 |
thy |
25073
13db30d367d2
locale pred: authentic syntax, tuned aprop_tr' accordingly;
wenzelm
parents:
25067
diff
changeset
|
1806 |
|> bodyT = propT ? Sign.add_advanced_trfuns ([], [], [aprop_tr' (length args) name], []) |
28110 | 1807 |
|> Sign.declare_const [] ((Name.binding bname, predT), NoSyn) |> snd |
27692 | 1808 |
|> PureThy.add_defs false |
27865
27a8ad9612a3
moved basic thm operations from structure PureThy to Thm (cf. more_thm.ML);
wenzelm
parents:
27761
diff
changeset
|
1809 |
[((Thm.def_name bname, Logic.mk_equals (head, body)), [Thm.kind_internal])]; |
20059 | 1810 |
val defs_ctxt = ProofContext.init defs_thy |> Variable.declare_term head; |
13394 | 1811 |
|
16458 | 1812 |
val cert = Thm.cterm_of defs_thy; |
13375 | 1813 |
|
20059 | 1814 |
val intro = Goal.prove_global defs_thy [] norm_ts statement (fn _ => |
21708 | 1815 |
MetaSimplifier.rewrite_goals_tac [pred_def] THEN |
13375 | 1816 |
Tactic.compose_tac (false, body_eq RS Drule.equal_elim_rule1, 1) 1 THEN |
23418 | 1817 |
Tactic.compose_tac (false, |
1818 |
Conjunction.intr_balanced (map (Thm.assume o cert) norm_ts), 0) 1); |
|
13375 | 1819 |
|
1820 |
val conjuncts = |
|
19423 | 1821 |
(Drule.equal_elim_rule2 OF [body_eq, |
21708 | 1822 |
MetaSimplifier.rewrite_rule [pred_def] (Thm.assume (cert statement))]) |
23418 | 1823 |
|> Conjunction.elim_balanced (length ts); |
17257
0ab67cb765da
introduced binding priority 1 for linear combinators etc.
haftmann
parents:
17228
diff
changeset
|
1824 |
val axioms = ts ~~ conjuncts |> map (fn (t, ax) => |
20059 | 1825 |
Element.prove_witness defs_ctxt t |
21708 | 1826 |
(MetaSimplifier.rewrite_goals_tac defs THEN |
13375 | 1827 |
Tactic.compose_tac (false, ax, 0) 1)); |
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1828 |
in ((statement, intro, axioms), defs_thy) end; |
13375 | 1829 |
|
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1830 |
fun assumes_to_notes (Assumes asms) axms = |
21441 | 1831 |
fold_map (fn (a, spec) => fn axs => |
1832 |
let val (ps, qs) = chop (length spec) axs |
|
1833 |
in ((a, [(ps, [])]), qs) end) asms axms |
|
1834 |
|> apfst (curry Notes Thm.assumptionK) |
|
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1835 |
| assumes_to_notes e axms = (e, axms); |
13394 | 1836 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1837 |
(* CB: the following two change only "new" elems, these have identifier ("", _). *) |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1838 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1839 |
(* turn Assumes into Notes elements *) |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1840 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1841 |
fun change_assumes_elemss axioms elemss = |
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1842 |
let |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1843 |
val satisfy = Element.morph_ctxt (Element.satisfy_morphism axioms); |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1844 |
fun change (id as ("", _), es) = |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1845 |
fold_map assumes_to_notes (map satisfy es) |
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1846 |
#-> (fn es' => pair (id, es')) |
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1847 |
| change e = pair e; |
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1848 |
in |
19780 | 1849 |
fst (fold_map change elemss (map Element.conclude_witness axioms)) |
18550
59b89f625d68
add_local_context now yields imported and body elements seperatly; additional slight clenup in code
haftmann
parents:
18546
diff
changeset
|
1850 |
end; |
13394 | 1851 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1852 |
(* adjust hyps of Notes elements *) |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1853 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1854 |
fun change_elemss_hyps axioms elemss = |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1855 |
let |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1856 |
val satisfy = Element.morph_ctxt (Element.satisfy_morphism axioms); |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
1857 |
fun change (id as ("", _), es) = (id, map (fn e as Notes _ => satisfy e | e => e) es) |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1858 |
| change e = e; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1859 |
in map change elemss end; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1860 |
|
13394 | 1861 |
in |
13375 | 1862 |
|
15104 | 1863 |
(* CB: main predicate definition function *) |
1864 |
||
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1865 |
fun define_preds pname (parms, ((exts, exts'), (ints, ints')), defs) elemss thy = |
13394 | 1866 |
let |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1867 |
val ((elemss', more_ts), a_elem, a_intro, thy'') = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1868 |
if null exts then ((elemss, []), [], [], thy) |
13394 | 1869 |
else |
1870 |
let |
|
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1871 |
val aname = if null ints then pname else pname ^ "_" ^ axiomsN; |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1872 |
val ((statement, intro, axioms), thy') = |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1873 |
thy |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1874 |
|> def_pred aname parms defs exts exts'; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1875 |
val elemss' = change_assumes_elemss axioms elemss; |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1876 |
val a_elem = [(("", []), |
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1877 |
[Assumes [((Name.binding (pname ^ "_" ^ axiomsN), []), [(statement, [])])]])]; |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1878 |
val (_, thy'') = |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1879 |
thy' |
27692 | 1880 |
|> Sign.add_path aname |
1881 |
|> Sign.no_base_names |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1882 |
|> PureThy.note_thmss Thm.internalK [((Name.binding introN, []), [([intro], [])])] |
27692 | 1883 |
||> Sign.restore_naming thy'; |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1884 |
in ((elemss', [statement]), a_elem, [intro], thy'') end; |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1885 |
val (predicate, stmt', elemss'', b_intro, thy'''') = |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1886 |
if null ints then (([], []), more_ts, elemss' @ a_elem, [], thy'') |
13394 | 1887 |
else |
1888 |
let |
|
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1889 |
val ((statement, intro, axioms), thy''') = |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1890 |
thy'' |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1891 |
|> def_pred pname parms defs (ints @ more_ts) (ints' @ more_ts); |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1892 |
val cstatement = Thm.cterm_of thy''' statement; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1893 |
val elemss'' = change_elemss_hyps axioms elemss'; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1894 |
val b_elem = [(("", []), |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1895 |
[Assumes [((Name.binding (pname ^ "_" ^ axiomsN), []), [(statement, [])])]])]; |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1896 |
val (_, thy'''') = |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1897 |
thy''' |
27692 | 1898 |
|> Sign.add_path pname |
1899 |
|> Sign.no_base_names |
|
1900 |
|> PureThy.note_thmss Thm.internalK |
|
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1901 |
[((Name.binding introN, []), [([intro], [])]), |
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1902 |
((Name.binding axiomsN, []), |
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
1903 |
[(map (Drule.standard o Element.conclude_witness) axioms, [])])] |
27692 | 1904 |
||> Sign.restore_naming thy'''; |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1905 |
in (([cstatement], axioms), [statement], elemss'' @ b_elem, [intro], thy'''') end; |
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
1906 |
in (((elemss'', predicate, stmt'), (a_intro, b_intro)), thy'''') end; |
13375 | 1907 |
|
1908 |
end; |
|
13336 | 1909 |
|
1910 |
||
13297 | 1911 |
(* add_locale(_i) *) |
1912 |
||
1913 |
local |
|
1914 |
||
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1915 |
(* turn Defines into Notes elements, accumulate definition terms *) |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1916 |
|
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1917 |
fun defines_to_notes is_ext thy (Defines defs) defns = |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1918 |
let |
28084
a05ca48ef263
type Attrib.binding abbreviates Name.binding without attributes;
wenzelm
parents:
28083
diff
changeset
|
1919 |
val defs' = map (fn (_, (def, _)) => (Attrib.no_binding, (def, []))) defs |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1920 |
val notes = map (fn (a, (def, _)) => |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1921 |
(a, [([assume (cterm_of thy def)], [])])) defs |
21441 | 1922 |
in |
1923 |
(if is_ext then SOME (Notes (Thm.definitionK, notes)) else NONE, defns @ [Defines defs']) |
|
1924 |
end |
|
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1925 |
| defines_to_notes _ _ e defns = (SOME e, defns); |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1926 |
|
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1927 |
fun change_defines_elemss thy elemss defns = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1928 |
let |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1929 |
fun change (id as (n, _), es) defns = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1930 |
let |
19942
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1931 |
val (es', defns') = fold_map (defines_to_notes (n="") thy) es defns |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1932 |
in ((id, map_filter I es'), defns') end |
dc92e3aebc71
Improved handling of defines imported in duplicate.
ballarin
parents:
19932
diff
changeset
|
1933 |
in fold_map change elemss defns end; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1934 |
|
18343 | 1935 |
fun gen_add_locale prep_ctxt prep_expr |
22573 | 1936 |
predicate_name bname raw_imports raw_body thy = |
27681 | 1937 |
(* predicate_name: "" - locale with predicate named as locale |
1938 |
"name" - locale with predicate named "name" *) |
|
13297 | 1939 |
let |
27681 | 1940 |
val thy_ctxt = ProofContext.init thy; |
16458 | 1941 |
val name = Sign.full_name thy bname; |
21962 | 1942 |
val _ = is_some (get_locale thy name) andalso |
1943 |
error ("Duplicate definition of locale " ^ quote name); |
|
13297 | 1944 |
|
17228 | 1945 |
val (((import_ctxt, import_elemss), (body_ctxt, body_elemss, syn)), |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1946 |
text as (parms, ((_, exts'), _), defs)) = |
27681 | 1947 |
prep_ctxt raw_imports raw_body thy_ctxt; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1948 |
val elemss = import_elemss @ body_elemss |> |
27681 | 1949 |
map_filter (fn ((id, Assumed axs), elems) => SOME (id, elems) | _ => NONE); |
13297 | 1950 |
|
23178 | 1951 |
val extraTs = List.foldr Term.add_term_tfrees [] exts' \\ |
1952 |
List.foldr Term.add_typ_tfrees [] (map snd parms); |
|
17228 | 1953 |
val _ = if null extraTs then () |
17437 | 1954 |
else warning ("Additional type variable(s) in locale specification " ^ quote bname); |
17228 | 1955 |
|
27681 | 1956 |
val predicate_name' = case predicate_name of "" => bname | _ => predicate_name; |
27692 | 1957 |
val (elemss', defns) = change_defines_elemss thy elemss []; |
1958 |
val elemss'' = elemss' @ [(("", []), defns)]; |
|
1959 |
val (((elemss''', predicate as (pred_statement, pred_axioms), stmt'), intros), thy') = |
|
1960 |
define_preds predicate_name' text elemss'' thy; |
|
1961 |
val regs = pred_axioms |
|
1962 |
|> fold_map (fn (id, elems) => fn wts => let |
|
1963 |
val ts = flat (map_filter (fn (Assumes asms) => |
|
1964 |
SOME (maps (map #1 o #2) asms) | _ => NONE) elems); |
|
1965 |
val (wts1, wts2) = chop (length ts) wts; |
|
1966 |
in ((apsnd (map fst) id, wts1), wts2) end) elemss''' |
|
1967 |
|> fst |
|
27681 | 1968 |
|> map_filter (fn (("", _), _) => NONE | e => SOME e); |
18137 | 1969 |
fun axiomify axioms elemss = |
15206
09d78ec709c7
Modified locales: improved implementation of "includes".
ballarin
parents:
15127
diff
changeset
|
1970 |
(axioms, elemss) |> foldl_map (fn (axs, (id, elems)) => let |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1971 |
val ts = flat (map_filter (fn (Assumes asms) => |
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
1972 |
SOME (maps (map #1 o #2) asms) | _ => NONE) elems); |
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
1973 |
val (axs1, axs2) = chop (length ts) axs; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
1974 |
in (axs2, ((id, Assumed axs1), elems)) end) |
27692 | 1975 |
|> snd; |
27681 | 1976 |
val ((_, facts), ctxt) = activate_facts true (K I) |
27692 | 1977 |
(axiomify pred_axioms elemss''') (ProofContext.init thy'); |
27681 | 1978 |
val view_ctxt = Assumption.add_view thy_ctxt pred_statement ctxt; |
26634
149f80f27c84
replaced Drule.close_derivation/Goal.close_result by Thm.close_derivation (removed obsolete compression);
wenzelm
parents:
26463
diff
changeset
|
1979 |
val export = Thm.close_derivation o Goal.norm_result o |
21602 | 1980 |
singleton (ProofContext.export view_ctxt thy_ctxt); |
13420 | 1981 |
val facts' = facts |> map (fn (a, ths) => ((a, []), [(map export ths, [])])); |
27692 | 1982 |
val elems' = maps #2 (filter (equal "" o #1 o #1) elemss'''); |
19783 | 1983 |
val elems'' = map_filter (fn (Fixes _) => NONE | e => SOME e) elems'; |
27681 | 1984 |
val axs' = map (Element.assume_witness thy') stmt'; |
1985 |
val loc_ctxt = thy' |
|
27692 | 1986 |
|> Sign.add_path bname |
1987 |
|> Sign.no_base_names |
|
1988 |
|> PureThy.note_thmss Thm.assumptionK facts' |> snd |
|
1989 |
|> Sign.restore_naming thy' |
|
27686 | 1990 |
|> register_locale name {axiom = axs', |
19783 | 1991 |
elems = map (fn e => (e, stamp ())) elems'', |
27692 | 1992 |
params = params_of elemss''' |> map (fn (x, SOME T) => ((x, T), the (Symtab.lookup syn x))), |
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
1993 |
decls = ([], []), |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
1994 |
regs = regs, |
25619 | 1995 |
intros = intros, |
27681 | 1996 |
dests = map Element.conclude_witness pred_axioms} |
21393
c648e24fd7ee
add_locale: re-init result context (avoids subtle modifications after introducing predicate views internally);
wenzelm
parents:
21370
diff
changeset
|
1997 |
|> init name; |
c648e24fd7ee
add_locale: re-init result context (avoids subtle modifications after introducing predicate views internally);
wenzelm
parents:
21370
diff
changeset
|
1998 |
in (name, loc_ctxt) end; |
13297 | 1999 |
|
2000 |
in |
|
2001 |
||
18917 | 2002 |
val add_locale = gen_add_locale read_context intern_expr; |
2003 |
val add_locale_i = gen_add_locale cert_context (K I); |
|
13297 | 2004 |
|
2005 |
end; |
|
2006 |
||
26463 | 2007 |
val _ = Context.>> (Context.map_theory |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
2008 |
(add_locale_i "" "var" empty [Fixes [(Name.binding (Name.internal "x"), NONE, NoSyn)]] #> |
20965 | 2009 |
snd #> ProofContext.theory_of #> |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
2010 |
add_locale_i "" "struct" empty [Fixes [(Name.binding (Name.internal "S"), NONE, Structure)]] #> |
26463 | 2011 |
snd #> ProofContext.theory_of)); |
15801 | 2012 |
|
13297 | 2013 |
|
12730 | 2014 |
|
17355 | 2015 |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2016 |
(** Normalisation of locale statements --- |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2017 |
discharges goals implied by interpretations **) |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2018 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2019 |
local |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2020 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2021 |
fun locale_assm_intros thy = |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2022 |
Symtab.fold (fn (_, {intros = (a, _), ...}) => fn intros => (a @ intros)) |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
2023 |
(#2 (LocalesData.get thy)) []; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2024 |
fun locale_base_intros thy = |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2025 |
Symtab.fold (fn (_, {intros = (_, b), ...}) => fn intros => (b @ intros)) |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
2026 |
(#2 (LocalesData.get thy)) []; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2027 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2028 |
fun all_witnesses ctxt = |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2029 |
let |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2030 |
val thy = ProofContext.theory_of ctxt; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2031 |
fun get registrations = Symtab.fold (fn (_, regs) => fn thms => |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2032 |
(Registrations.dest thy regs |> map (fn (_, (_, (exp, _), wits, _)) => |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2033 |
map (Element.conclude_witness #> Morphism.thm exp) wits) |> flat) @ thms) |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2034 |
registrations []; |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
2035 |
in get (RegistrationsData.get (Context.Proof ctxt)) end; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2036 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2037 |
in |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2038 |
|
19984
29bb4659f80a
Method intro_locales replaced by intro_locales and unfold_locales.
ballarin
parents:
19942
diff
changeset
|
2039 |
fun intro_locales_tac eager ctxt facts st = |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2040 |
let |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2041 |
val wits = all_witnesses ctxt; |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2042 |
val thy = ProofContext.theory_of ctxt; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2043 |
val intros = locale_base_intros thy @ (if eager then locale_assm_intros thy else []); |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2044 |
in |
25270 | 2045 |
Method.intros_tac (wits @ intros) facts st |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2046 |
end; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2047 |
|
26463 | 2048 |
val _ = Context.>> (Context.map_theory |
2049 |
(Method.add_methods |
|
2050 |
[("intro_locales", |
|
2051 |
Method.ctxt_args (fn ctxt => Method.METHOD (intro_locales_tac false ctxt)), |
|
2052 |
"back-chain introduction rules of locales without unfolding predicates"), |
|
2053 |
("unfold_locales", |
|
2054 |
Method.ctxt_args (fn ctxt => Method.METHOD (intro_locales_tac true ctxt)), |
|
2055 |
"back-chain all introduction rules of locales")])); |
|
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2056 |
|
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2057 |
end; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2058 |
|
19780 | 2059 |
|
15598
4ab52355bb53
Registrations of global locale interpretations: improved, better naming.
ballarin
parents:
15596
diff
changeset
|
2060 |
(** Interpretation commands **) |
15596 | 2061 |
|
2062 |
local |
|
2063 |
||
2064 |
(* extract proof obligations (assms and defs) from elements *) |
|
2065 |
||
19780 | 2066 |
fun extract_asms_elems ((id, Assumed _), elems) = (id, maps Element.prems_of elems) |
17138 | 2067 |
| extract_asms_elems ((id, Derived _), _) = (id, []); |
15596 | 2068 |
|
2069 |
||
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
2070 |
(* activate instantiated facts in theory or context *) |
15596 | 2071 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2072 |
fun gen_activate_facts_elemss mk_ctxt note note_interp attrib put_reg add_wit add_eqn |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2073 |
prfx all_elemss pss propss eq_attns (exp, imp) thmss thy_ctxt = |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2074 |
let |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2075 |
val ctxt = mk_ctxt thy_ctxt; |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2076 |
fun get_reg thy_ctxt = get_local_registration (mk_ctxt thy_ctxt); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2077 |
fun test_reg thy_ctxt = test_local_registration (mk_ctxt thy_ctxt); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2078 |
|
28005 | 2079 |
val (all_propss, eq_props) = chop (length all_elemss) propss; |
2080 |
val (all_thmss, eq_thms) = chop (length all_elemss) thmss; |
|
27761
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2081 |
|
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2082 |
(* Filter out fragments already registered. *) |
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2083 |
|
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2084 |
val (new_elemss, xs) = split_list (filter_out (fn (((id, _), _), _) => |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2085 |
test_reg thy_ctxt id) (all_elemss ~~ (pss ~~ (all_propss ~~ all_thmss)))); |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2086 |
val (new_pss, ys) = split_list xs; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2087 |
val (new_propss, new_thmss) = split_list ys; |
17033 | 2088 |
|
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2089 |
val thy_ctxt' = thy_ctxt |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2090 |
(* add registrations *) |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2091 |
|> fold (fn (((id, _), _), ps) => put_reg id (prfx, param_prefix ps) (exp, imp)) (new_elemss ~~ new_pss) |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2092 |
(* add witnesses of Assumed elements (only those generate proof obligations) *) |
28005 | 2093 |
|> fold (fn (id, thms) => fold (add_wit id) thms) (map fst new_propss ~~ new_thmss) |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2094 |
(* add equations *) |
24693 | 2095 |
|> fold (fn (id, thms) => fold (add_eqn id) thms) (map fst eq_props ~~ |
24952
f336c36f41a0
removed redundant strip_vars/abs_eqn, use improved Drule.abs_def instead;
wenzelm
parents:
24941
diff
changeset
|
2096 |
(map o map) (Drule.abs_def o LocalDefs.meta_rewrite_rule ctxt o |
23918 | 2097 |
Element.conclude_witness) eq_thms); |
15596 | 2098 |
|
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2099 |
val prems = flat (map_filter |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2100 |
(fn ((id, Assumed _), _) => Option.map #2 (get_reg thy_ctxt' imp id) |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2101 |
| ((_, Derived _), _) => NONE) all_elemss); |
27761
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2102 |
|
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2103 |
val thy_ctxt'' = thy_ctxt' |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2104 |
(* add witnesses of Derived elements *) |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2105 |
|> fold (fn (id, thms) => fold (add_wit id o Element.morph_witness (Element.satisfy_morphism prems)) thms) |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2106 |
(map_filter (fn ((_, Assumed _), _) => NONE |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2107 |
| ((id, Derived thms), _) => SOME (id, thms)) new_elemss) |
19780 | 2108 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2109 |
fun activate_elem inst loc prfx pprfx (Notes (kind, facts)) thy_ctxt = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2110 |
let |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2111 |
val ctxt = mk_ctxt thy_ctxt; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2112 |
val facts' = facts |> |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2113 |
interpret_args (ProofContext.theory_of ctxt) inst exp (attrib thy_ctxt) |> |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2114 |
add_param_prefixss pprfx; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2115 |
in snd (note_interp kind loc prfx facts' thy_ctxt) end |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2116 |
| activate_elem _ _ _ _ _ thy_ctxt = thy_ctxt; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2117 |
|
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2118 |
fun activate_elems ((((loc, ext_ts), _), _), ps) thy_ctxt = |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2119 |
let |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2120 |
val ctxt = mk_ctxt thy_ctxt; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2121 |
val thy = ProofContext.theory_of ctxt; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2122 |
val {params, elems, ...} = the_locale thy loc; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2123 |
val parms = map fst params; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2124 |
val pprfx = param_prefix ps; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2125 |
val ids = flatten (ProofContext.init thy, intern_expr thy) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2126 |
(([], Symtab.empty), Expr (Locale loc)) |> fst |> fst; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2127 |
val (insts, prems, eqns) = collect_witnesses ctxt imp parms ids ext_ts; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2128 |
val inst = inst_morph thy (snd prfx) pprfx insts prems eqns; |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2129 |
in |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2130 |
fold (activate_elem inst loc prfx pprfx) (map fst elems) thy_ctxt |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2131 |
end; |
27761
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2132 |
|
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2133 |
in |
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2134 |
thy_ctxt'' |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2135 |
(* add equations as lemmas to context *) |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2136 |
|> fold (fn (attns, thms) => |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2137 |
fold (fn (attn, thm) => note "lemma" |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2138 |
[(apsnd (map (attrib thy_ctxt'')) attn, |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2139 |
[([Element.conclude_witness thm], [])])] #> snd) |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2140 |
(attns ~~ thms)) (unflat eq_thms eq_attns ~~ eq_thms) |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2141 |
(* add interpreted facts *) |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2142 |
|> fold activate_elems (new_elemss ~~ new_pss) |
21499
fbd6422a847a
uniform interface for type_syntax/term_syntax/declaration, dependent on morphism;
wenzelm
parents:
21483
diff
changeset
|
2143 |
end; |
15596 | 2144 |
|
17355 | 2145 |
fun global_activate_facts_elemss x = gen_activate_facts_elemss |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2146 |
ProofContext.init |
27692 | 2147 |
PureThy.note_thmss |
21441 | 2148 |
global_note_prefix_i |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2149 |
Attrib.attribute_i |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2150 |
put_global_registration |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2151 |
add_global_witness |
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2152 |
add_global_equation |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2153 |
x; |
17355 | 2154 |
|
2155 |
fun local_activate_facts_elemss x = gen_activate_facts_elemss |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2156 |
I |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2157 |
ProofContext.note_thmss_i |
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
2158 |
local_note_prefix_i |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2159 |
(Attrib.attribute_i o ProofContext.theory_of) |
17033 | 2160 |
put_local_registration |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2161 |
add_local_witness |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2162 |
add_local_equation |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2163 |
x; |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2164 |
|
25067
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2165 |
fun prep_instantiations parse_term parse_prop ctxt parms (insts, eqns) = |
15596 | 2166 |
let |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2167 |
(* parameters *) |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2168 |
val (parm_names, parm_types) = parms |> split_list |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2169 |
||> map (TypeInfer.paramify_vars o Logic.varifyT); |
25038 | 2170 |
val type_parms = fold Term.add_tvarsT parm_types [] |> map (Logic.mk_type o TVar); |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2171 |
val type_parm_names = fold Term.add_tfreesT (map snd parms) [] |> map fst; |
22772
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2172 |
|
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2173 |
(* parameter instantiations *) |
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2174 |
val d = length parms - length insts; |
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2175 |
val insts = |
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2176 |
if d < 0 then error "More arguments than parameters in instantiation." |
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2177 |
else insts @ replicate d NONE; |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2178 |
val (given_ps, given_insts) = |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2179 |
((parm_names ~~ parm_types) ~~ insts) |> map_filter |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2180 |
(fn (_, NONE) => NONE |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2181 |
| ((n, T), SOME inst) => SOME ((n, T), inst)) |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2182 |
|> split_list; |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2183 |
val (given_parm_names, given_parm_types) = given_ps |> split_list; |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2184 |
|
25067
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2185 |
(* parse insts / eqns *) |
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2186 |
val given_insts' = map (parse_term ctxt) given_insts; |
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2187 |
val eqns' = map (parse_prop ctxt) eqns; |
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2188 |
|
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2189 |
(* type inference and contexts *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2190 |
val arg = type_parms @ map2 TypeInfer.constrain given_parm_types given_insts' @ eqns'; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2191 |
val res = Syntax.check_terms ctxt arg; |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2192 |
val ctxt' = ctxt |> fold Variable.auto_fixes res; |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2193 |
|
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2194 |
(* instantiation *) |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2195 |
val (type_parms'', res') = chop (length type_parms) res; |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2196 |
val (given_insts'', eqns'') = chop (length given_insts) res'; |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2197 |
val instT = Symtab.make (type_parm_names ~~ map Logic.dest_type type_parms''); |
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2198 |
val inst = Symtab.make (given_parm_names ~~ given_insts''); |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2199 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2200 |
(* export from eigencontext *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2201 |
val export = Variable.export_morphism ctxt' ctxt; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2202 |
|
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2203 |
(* import, its inverse *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2204 |
val domT = fold Term.add_tfrees res [] |> map TFree; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2205 |
val importT = domT |> map (fn x => (Morphism.typ export x, x)) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2206 |
|> map_filter (fn (TFree _, _) => NONE (* fixed point of export *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2207 |
| (TVar y, x) => SOME (fst y, x) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2208 |
| _ => error "internal: illegal export in interpretation") |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2209 |
|> Vartab.make; |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2210 |
val dom = fold Term.add_frees res [] |> map Free; |
25357
6ea18fd11058
avoid "import" as identifier, which is a keyword in Alice;
wenzelm
parents:
25286
diff
changeset
|
2211 |
val imprt = dom |> map (fn x => (Morphism.term export x, x)) |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2212 |
|> map_filter (fn (Free _, _) => NONE (* fixed point of export *) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2213 |
| (Var y, x) => SOME (fst y, x) |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2214 |
| _ => error "internal: illegal export in interpretation") |
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2215 |
|> Vartab.make; |
25357
6ea18fd11058
avoid "import" as identifier, which is a keyword in Alice;
wenzelm
parents:
25286
diff
changeset
|
2216 |
in (((instT, inst), eqns''), (export, ((importT, domT), (imprt, dom)))) end; |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2217 |
|
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2218 |
val read_instantiations = prep_instantiations Syntax.parse_term Syntax.parse_prop; |
25067
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2219 |
val check_instantiations = prep_instantiations (K I) (K I); |
15598
4ab52355bb53
Registrations of global locale interpretations: improved, better naming.
ballarin
parents:
15596
diff
changeset
|
2220 |
|
22772
e0788ff2e811
read_instantiations: proper type-inference with fixed variables, infer parameter types as well;
wenzelm
parents:
22756
diff
changeset
|
2221 |
fun gen_prep_registration mk_ctxt test_reg activate |
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2222 |
prep_attr prep_expr prep_insts |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
2223 |
thy_ctxt prfx raw_expr raw_insts = |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2224 |
let |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2225 |
val ctxt = mk_ctxt thy_ctxt; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2226 |
val thy = ProofContext.theory_of ctxt; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2227 |
val ctxt' = ProofContext.init thy; |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2228 |
fun prep_attn attn = (apsnd o map) |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2229 |
(Attrib.crude_closure ctxt o Args.assignable o prep_attr thy) attn; |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2230 |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2231 |
val expr = prep_expr thy raw_expr; |
15596 | 2232 |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2233 |
val pts = params_of_expr ctxt' [] expr ([], Symtab.empty, Symtab.empty); |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2234 |
val params_ids = make_params_ids (#1 pts); |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2235 |
val raw_params_elemss = make_raw_params_elemss pts; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2236 |
val ((ids, _), raw_elemss) = flatten (ctxt', I) (([], Symtab.empty), Expr expr); |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2237 |
val ((parms, all_elemss, _), (_, (_, defs, _))) = |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2238 |
read_elemss false ctxt' [] (raw_params_elemss @ raw_elemss) []; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2239 |
|
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2240 |
(** compute instantiation **) |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2241 |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2242 |
(* consistency check: equations need to be stored in a particular locale, |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2243 |
therefore if equations are present locale expression must be a name *) |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2244 |
|
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2245 |
val _ = case (expr, snd raw_insts) of |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2246 |
(Locale _, _) => () | (_, []) => () |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2247 |
| (_, _) => error "Interpretations with `where' only permitted if locale expression is a name."; |
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2248 |
|
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2249 |
(* read or certify instantiation *) |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2250 |
val (raw_insts', raw_eqns) = raw_insts; |
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2251 |
val (raw_eq_attns, raw_eqns') = split_list raw_eqns; |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2252 |
val (((instT, inst1), eqns), morphs) = prep_insts ctxt parms (raw_insts', raw_eqns'); |
25095
ea8307dac208
Interpretation equations may have name and/or attribute;
ballarin
parents:
25073
diff
changeset
|
2253 |
val eq_attns = map prep_attn raw_eq_attns; |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2254 |
|
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2255 |
(* defined params without given instantiation *) |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2256 |
val not_given = filter_out (Symtab.defined inst1 o fst) parms; |
18137 | 2257 |
fun add_def (p, pT) inst = |
15596 | 2258 |
let |
2259 |
val (t, T) = case find_first (fn (Free (a, _), _) => a = p) defs of |
|
2260 |
NONE => error ("Instance missing for parameter " ^ quote p) |
|
2261 |
| SOME (Free (_, T), t) => (t, T); |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2262 |
val d = Element.inst_term (instT, inst) t; |
18137 | 2263 |
in Symtab.update_new (p, d) inst end; |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2264 |
val inst2 = fold add_def not_given inst1; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2265 |
val inst_morphism = Element.inst_morphism thy (instT, inst2); |
18137 | 2266 |
(* Note: insts contain no vars. *) |
15596 | 2267 |
|
2268 |
(** compute proof obligations **) |
|
2269 |
||
15598
4ab52355bb53
Registrations of global locale interpretations: improved, better naming.
ballarin
parents:
15596
diff
changeset
|
2270 |
(* restore "small" ids *) |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2271 |
val ids' = map (fn ((n, ps), (_, mode)) => |
19783 | 2272 |
((n, map (fn p => Free (p, (the o AList.lookup (op =) parms) p)) ps), mode)) |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2273 |
ids; |
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2274 |
val (_, all_elemss') = chop (length raw_params_elemss) all_elemss |
15596 | 2275 |
(* instantiate ids and elements *) |
19931
fb32b43e7f80
Restructured locales with predicates: import is now an interpretation.
ballarin
parents:
19914
diff
changeset
|
2276 |
val inst_elemss = (ids' ~~ all_elemss') |> map (fn (((n, ps), _), ((_, mode), elems)) => |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2277 |
((n, map (Morphism.term (inst_morphism $> fst morphs)) ps), |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
2278 |
map (fn Int e => Element.morph_ctxt inst_morphism e) elems) |
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
2279 |
|> apfst (fn id => (id, map_mode (map (Element.morph_witness inst_morphism)) mode))); |
28053 | 2280 |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2281 |
(* equations *) |
23918 | 2282 |
val eqn_elems = if null eqns then [] |
2283 |
else [(Library.last_elem inst_elemss |> fst |> fst, eqns)]; |
|
22658
263d42253f53
Experimental interpretation code for definitions.
ballarin
parents:
22573
diff
changeset
|
2284 |
|
27761
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2285 |
val propss = map extract_asms_elems inst_elemss @ eqn_elems; |
b95e9ba0ca1d
Interpretation command (theory/proof context) no longer simplifies goal.
ballarin
parents:
27716
diff
changeset
|
2286 |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2287 |
in (propss, activate prfx inst_elemss (map (snd o fst) ids) propss eq_attns morphs) end; |
15596 | 2288 |
|
22756 | 2289 |
fun gen_prep_global_registration mk_ctxt = gen_prep_registration ProofContext.init |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2290 |
test_global_registration |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2291 |
global_activate_facts_elemss mk_ctxt; |
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
2292 |
|
22756 | 2293 |
fun gen_prep_local_registration mk_ctxt = gen_prep_registration I |
24787
df56433cc059
Theory/context data restructured; simplified interface for printing of interpretations.
ballarin
parents:
24751
diff
changeset
|
2294 |
test_local_registration |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2295 |
local_activate_facts_elemss mk_ctxt; |
15624
484178635bd8
Further work on interpretation commands. New command `interpret' for
ballarin
parents:
15623
diff
changeset
|
2296 |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2297 |
val prep_global_registration = gen_prep_global_registration |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2298 |
Attrib.intern_src intern_expr read_instantiations; |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2299 |
val prep_global_registration_i = gen_prep_global_registration |
25067
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2300 |
(K I) (K I) check_instantiations; |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2301 |
|
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2302 |
val prep_local_registration = gen_prep_local_registration |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2303 |
Attrib.intern_src intern_expr read_instantiations; |
24941
9ab032df81c8
Prepare proper interface of interpretation_i, interpret_i.
ballarin
parents:
24920
diff
changeset
|
2304 |
val prep_local_registration_i = gen_prep_local_registration |
25067
0f19e65ac0b6
clarified naming conventions of 'parse' and 'check' (as opposed to former 'cert');
wenzelm
parents:
25038
diff
changeset
|
2305 |
(K I) (K I) check_instantiations; |
15596 | 2306 |
|
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2307 |
fun prep_registration_in_locale target expr thy = |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2308 |
(* target already in internal form *) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2309 |
let |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2310 |
val ctxt = ProofContext.init thy; |
17138 | 2311 |
val ((raw_target_ids, target_syn), _) = flatten (ctxt, I) |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2312 |
(([], Symtab.empty), Expr (Locale target)); |
19278 | 2313 |
val fixed = the_locale thy target |> #params |> map #1; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2314 |
val ((all_ids, syn), raw_elemss) = flatten (ctxt, intern_expr thy) |
17138 | 2315 |
((raw_target_ids, target_syn), Expr expr); |
19018
88b4979193d8
added abbreviations: activated by init, no expressions yet;
wenzelm
parents:
18964
diff
changeset
|
2316 |
val (target_ids, ids) = chop (length raw_target_ids) all_ids; |
17138 | 2317 |
val ((parms, elemss, _), _) = read_elemss false ctxt fixed raw_elemss []; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2318 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2319 |
(** compute proof obligations **) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2320 |
|
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2321 |
(* restore "small" ids, with mode *) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2322 |
val ids' = map (apsnd snd) ids; |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2323 |
(* remove Int markers *) |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2324 |
val elemss' = map (fn (_, es) => |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2325 |
map (fn Int e => e) es) elemss |
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2326 |
(* extract assumptions and defs *) |
17138 | 2327 |
val ids_elemss = ids' ~~ elemss'; |
19780 | 2328 |
val propss = map extract_asms_elems ids_elemss; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2329 |
|
17138 | 2330 |
(** activation function: |
2331 |
- add registrations to the target locale |
|
2332 |
- add induced registrations for all global registrations of |
|
2333 |
the target, unless already present |
|
2334 |
- add facts of induced registrations to theory **) |
|
2335 |
||
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2336 |
fun activate thmss thy = let |
19780 | 2337 |
val satisfy = Element.satisfy_thm (flat thmss); |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2338 |
val ids_elemss_thmss = ids_elemss ~~ thmss; |
17138 | 2339 |
val regs = get_global_registrations thy target; |
2340 |
||
2341 |
fun activate_id (((id, Assumed _), _), thms) thy = |
|
17033 | 2342 |
thy |> put_registration_in_locale target id |
17138 | 2343 |
|> fold (add_witness_in_locale target id) thms |
2344 |
| activate_id _ thy = thy; |
|
2345 |
||
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2346 |
fun activate_reg (ext_ts, (((fully_qualified, prfx), pprfx), (exp, imp), _, _)) thy = |
21483
e4be91feca50
replaced Args.map_values/Element.map_ctxt_values by general morphism application;
wenzelm
parents:
21441
diff
changeset
|
2347 |
let |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2348 |
val (insts, wits, _) = collect_witnesses (ProofContext.init thy) imp fixed target_ids ext_ts; |
18137 | 2349 |
fun inst_parms ps = map |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2350 |
(the o AList.lookup (op =) (map #1 fixed ~~ ext_ts)) ps; |
19780 | 2351 |
val disch = Element.satisfy_thm wits; |
19482
9f11af8f7ef9
tuned basic list operators (flat, maps, map_filter);
wenzelm
parents:
19423
diff
changeset
|
2352 |
val new_elemss = filter (fn (((name, ps), _), _) => |
17138 | 2353 |
not (test_global_registration thy (name, inst_parms ps))) (ids_elemss); |
2354 |
fun activate_assumed_id (((_, Derived _), _), _) thy = thy |
|
2355 |
| activate_assumed_id ((((name, ps), Assumed _), _), thms) thy = let |
|
2356 |
val ps' = inst_parms ps; |
|
2357 |
in |
|
2358 |
if test_global_registration thy (name, ps') |
|
2359 |
then thy |
|
2360 |
else thy |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2361 |
|> put_global_registration (name, ps') ((fully_qualified, prfx), param_prefix ps) (exp, imp) |
19780 | 2362 |
|> fold (fn witn => fn thy => add_global_witness (name, ps') |
25286
35e954ff67f8
Use of export rather than standard in interpretation.
ballarin
parents:
25270
diff
changeset
|
2363 |
(Element.morph_witness (Element.inst_morphism thy insts) witn) thy) thms |
17138 | 2364 |
end; |
2365 |
||
2366 |
fun activate_derived_id ((_, Assumed _), _) thy = thy |
|
2367 |
| activate_derived_id (((name, ps), Derived ths), _) thy = let |
|
2368 |
val ps' = inst_parms ps; |
|
2369 |
in |
|
2370 |
if test_global_registration thy (name, ps') |
|
2371 |
then thy |
|
2372 |
else thy |
|
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2373 |
|> put_global_registration (name, ps') ((fully_qualified, prfx), param_prefix ps) (exp, imp) |
19780 | 2374 |
|> fold (fn witn => fn thy => add_global_witness (name, ps') |
2375 |
(witn |> Element.map_witness (fn (t, th) => (* FIXME *) |
|
18137 | 2376 |
(Element.inst_term insts t, |
19780 | 2377 |
disch (Element.inst_thm thy insts (satisfy th))))) thy) ths |
17138 | 2378 |
end; |
2379 |
||
26645
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
2380 |
fun activate_elem (loc, ps) (Notes (kind, facts)) thy = |
17138 | 2381 |
let |
21523 | 2382 |
val att_morphism = |
28107 | 2383 |
Morphism.name_morphism (Name.qualified prfx) $> |
28236
c447b60d67f5
Clearer separation of interpretation frontend and backend.
ballarin
parents:
28110
diff
changeset
|
2384 |
(* FIXME? treatment of parameter prefix *) |
21523 | 2385 |
Morphism.thm_morphism satisfy $> |
2386 |
Element.inst_morphism thy insts $> |
|
2387 |
Morphism.thm_morphism disch; |
|
17138 | 2388 |
val facts' = facts |
21523 | 2389 |
|> Attrib.map_facts (Attrib.attribute_i thy o Args.morph_values att_morphism) |
2390 |
|> map (apsnd (map (apfst (map (disch o Element.inst_thm thy insts o satisfy))))) |
|
17138 | 2391 |
in |
18377 | 2392 |
thy |
28053 | 2393 |
|> global_note_prefix_i kind loc (fully_qualified, prfx) facts' |
18377 | 2394 |
|> snd |
17138 | 2395 |
end |
26645
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
2396 |
| activate_elem _ _ thy = thy; |
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
2397 |
|
e114be97befe
Changed naming scheme for theorems generated by interpretations.
ballarin
parents:
26634
diff
changeset
|
2398 |
fun activate_elems ((id, _), elems) thy = fold (activate_elem id) elems thy; |
17138 | 2399 |
|
2400 |
in thy |> fold activate_assumed_id ids_elemss_thmss |
|
2401 |
|> fold activate_derived_id ids_elemss |
|
2402 |
|> fold activate_elems new_elemss end; |
|
17033 | 2403 |
in |
17138 | 2404 |
thy |> fold activate_id ids_elemss_thmss |
2405 |
|> fold activate_reg regs |
|
17033 | 2406 |
end; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2407 |
|
17033 | 2408 |
in (propss, activate) end; |
17000
552df70f52c2
First version of interpretation in locales. Not yet fully functional.
ballarin
parents:
16947
diff
changeset
|
2409 |
|
21005 | 2410 |
fun prep_propp propss = propss |> map (fn (_, props) => |
21361 | 2411 |
map (rpair [] o Element.mark_witness) props); |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2412 |
|
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2413 |
fun prep_result propps thmss = |
19780 | 2414 |
ListPair.map (fn ((_, props), thms) => map2 Element.make_witness props thms) (propps, thmss); |
17437 | 2415 |
|
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
2416 |
fun gen_interpretation prep_registration after_qed prfx raw_expr raw_insts thy = |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
2417 |
(* prfx = (flag indicating full qualification, name prefix) *) |
17355 | 2418 |
let |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
2419 |
val (propss, activate) = prep_registration thy prfx raw_expr raw_insts; |
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
2420 |
fun after_qed' results = |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
2421 |
ProofContext.theory (activate (prep_result propss results)) |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
2422 |
#> after_qed; |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2423 |
in |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2424 |
thy |
23418 | 2425 |
|> ProofContext.init |
21441 | 2426 |
|> Proof.theorem_i NONE after_qed' (prep_propp propss) |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2427 |
|> Element.refine_witness |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2428 |
|> Seq.hd |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2429 |
end; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2430 |
|
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
2431 |
fun gen_interpret prep_registration after_qed prfx expr insts int state = |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
2432 |
(* prfx = (flag indicating full qualification, name prefix) *) |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2433 |
let |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2434 |
val _ = Proof.assert_forward_or_chain state; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2435 |
val ctxt = Proof.context_of state; |
28085
914183e229e9
Interpretation commands no longer accept interpretation attributes.
ballarin
parents:
28084
diff
changeset
|
2436 |
val (propss, activate) = prep_registration ctxt prfx expr insts; |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2437 |
fun after_qed' results = |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2438 |
Proof.map_context (K (ctxt |> activate (prep_result propss results))) |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2439 |
#> Proof.put_facts NONE |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2440 |
#> after_qed; |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2441 |
in |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2442 |
state |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2443 |
|> Proof.local_goal (ProofDisplay.print_results int) (K I) ProofContext.bind_propp_i |
28083
103d9282a946
explicit type Name.binding for higher-specification elements;
wenzelm
parents:
28053
diff
changeset
|
2444 |
"interpret" NONE after_qed' (map (pair (Name.no_binding, [])) (prep_propp propss)) |
19810 | 2445 |
|> Element.refine_witness |> Seq.hd |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2446 |
end; |
17355 | 2447 |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2448 |
in |
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2449 |
|
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
2450 |
val interpretation_i = gen_interpretation prep_global_registration_i; |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2451 |
val interpretation = gen_interpretation prep_global_registration; |
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
2452 |
|
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2453 |
|
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
2454 |
fun interpretation_in_locale after_qed (raw_target, expr) thy = |
17355 | 2455 |
let |
2456 |
val target = intern thy raw_target; |
|
2457 |
val (propss, activate) = prep_registration_in_locale target expr thy; |
|
21361 | 2458 |
val raw_propp = prep_propp propss; |
21005 | 2459 |
|
2460 |
val (_, _, goal_ctxt, propp) = thy |
|
21665
ba07e24dc941
encode declarations as notes (attributes), which enables proper inheritance, interpretation etc.;
wenzelm
parents:
21602
diff
changeset
|
2461 |
|> ProofContext.init |
21361 | 2462 |
|> cert_context_statement (SOME target) [] raw_propp; |
21005 | 2463 |
|
2464 |
fun after_qed' results = |
|
20366
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
2465 |
ProofContext.theory (activate (prep_result propss results)) |
867696dc64fc
global goals/qeds: after_qed operates on Proof.context (potentially local_theory);
wenzelm
parents:
20317
diff
changeset
|
2466 |
#> after_qed; |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2467 |
in |
21005 | 2468 |
goal_ctxt |
21441 | 2469 |
|> Proof.theorem_i NONE after_qed' propp |
19810 | 2470 |
|> Element.refine_witness |> Seq.hd |
18123
1bb572e8cee9
avoid prove_plain, export_plain, simplified after_qed;
wenzelm
parents:
18038
diff
changeset
|
2471 |
end; |
17449
429ca1e21289
interpretation: use goal commands without target -- no storing of results;
wenzelm
parents:
17438
diff
changeset
|
2472 |
|
22351
587845efb4cf
locale: add_locale accepts explicit predicate name, interpretation supports non-mandatory prefixes
haftmann
parents:
22339
diff
changeset
|
2473 |
val interpret_i = gen_interpret prep_local_registration_i; |
22300
596f49b70c70
internal interfaces for interpretation and interpret
haftmann
parents:
22241
diff
changeset
|
2474 |
val interpret = gen_interpret prep_local_registration; |
15596 | 2475 |
|
11896 | 2476 |
end; |
17355 | 2477 |
|
2478 |
end; |