author | wenzelm |
Mon, 24 Oct 2022 20:37:32 +0200 | |
changeset 76371 | 1ac2416e8432 |
parent 74561 | 8e6c973003c8 |
child 77723 | b761c91c2447 |
permissions | -rw-r--r-- |
47308 | 1 |
(* Title: HOL/Tools/Lifting/lifting_info.ML |
2 |
Author: Ondrej Kuncar |
|
3 |
||
4 |
Context data for the lifting package. |
|
5 |
*) |
|
6 |
||
7 |
signature LIFTING_INFO = |
|
8 |
sig |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
9 |
type quot_map = {rel_quot_thm: thm} |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
10 |
val lookup_quot_maps: Proof.context -> string -> quot_map option |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
11 |
val print_quot_maps: Proof.context -> unit |
69089 | 12 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
13 |
type pcr = {pcrel_def: thm, pcr_cr_eq: thm} |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
14 |
type quotient = {quot_thm: thm, pcr_info: pcr option} |
53651 | 15 |
val pcr_eq: pcr * pcr -> bool |
16 |
val quotient_eq: quotient * quotient -> bool |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
17 |
val transform_quotient: morphism -> quotient -> quotient |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
18 |
val lookup_quotients: Proof.context -> string -> quotient option |
60235
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
19 |
val lookup_quot_thm_quotients: Proof.context -> thm -> quotient option |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
20 |
val update_quotients: string -> quotient -> Context.generic -> Context.generic |
53650 | 21 |
val delete_quotients: thm -> Context.generic -> Context.generic |
47308 | 22 |
val print_quotients: Proof.context -> unit |
23 |
||
53651 | 24 |
type restore_data = {quotient : quotient, transfer_rules: thm Item_Net.T} |
25 |
val lookup_restore_data: Proof.context -> string -> restore_data option |
|
26 |
val init_restore_data: string -> quotient -> Context.generic -> Context.generic |
|
69089 | 27 |
val add_transfer_rules_in_restore_data: string -> thm Item_Net.T -> Context.generic -> Context.generic |
53651 | 28 |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
29 |
val get_relator_eq_onp_rules: Proof.context -> thm list |
69089 | 30 |
|
47982
7aa35601ff65
prove reflexivity also for the quotient composition relation; reflp_preserve renamed to reflexivity_rule
kuncar
parents:
47951
diff
changeset
|
31 |
val get_reflexivity_rules: Proof.context -> thm list |
7aa35601ff65
prove reflexivity also for the quotient composition relation; reflp_preserve renamed to reflexivity_rule
kuncar
parents:
47951
diff
changeset
|
32 |
val add_reflexivity_rule_attribute: attribute |
47634
091bcd569441
hide the invariant constant for relators: invariant_commute infrastracture
kuncar
parents:
47308
diff
changeset
|
33 |
|
69089 | 34 |
type relator_distr_data = {pos_mono_rule: thm, neg_mono_rule: thm, |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
35 |
pos_distr_rules: thm list, neg_distr_rules: thm list} |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
36 |
val lookup_relator_distr_data: Proof.context -> string -> relator_distr_data option |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
37 |
|
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
38 |
val add_no_code_type: string -> Context.generic -> Context.generic |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
39 |
val is_no_code_type: Proof.context -> string -> bool |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
40 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
41 |
val get_quot_maps : Proof.context -> quot_map Symtab.table |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
42 |
val get_quotients : Proof.context -> quotient Symtab.table |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
43 |
val get_relator_distr_data : Proof.context -> relator_distr_data Symtab.table |
53651 | 44 |
val get_restore_data : Proof.context -> restore_data Symtab.table |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
45 |
val get_no_code_types : Proof.context -> unit Symtab.table |
53651 | 46 |
end |
47308 | 47 |
|
48 |
structure Lifting_Info: LIFTING_INFO = |
|
49 |
struct |
|
50 |
||
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
51 |
open Lifting_Util |
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
52 |
|
69089 | 53 |
|
54 |
(* context data *) |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
55 |
|
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
56 |
type quot_map = {rel_quot_thm: thm} |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
57 |
type pcr = {pcrel_def: thm, pcr_cr_eq: thm} |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
58 |
type quotient = {quot_thm: thm, pcr_info: pcr option} |
69089 | 59 |
type relator_distr_data = {pos_mono_rule: thm, neg_mono_rule: thm, |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
60 |
pos_distr_rules: thm list, neg_distr_rules: thm list} |
53651 | 61 |
type restore_data = {quotient : quotient, transfer_rules: thm Item_Net.T} |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
62 |
|
53684 | 63 |
fun pcr_eq ({pcrel_def = pcrel_def1, pcr_cr_eq = pcr_cr_eq1}, |
69089 | 64 |
{pcrel_def = pcrel_def2, pcr_cr_eq = pcr_cr_eq2}) = |
53684 | 65 |
Thm.eq_thm (pcrel_def1, pcrel_def2) andalso Thm.eq_thm (pcr_cr_eq1, pcr_cr_eq2) |
66 |
||
67 |
fun quotient_eq ({quot_thm = quot_thm1, pcr_info = pcr_info1}, |
|
68 |
{quot_thm = quot_thm2, pcr_info = pcr_info2}) = |
|
69088 | 69 |
Thm.eq_thm (quot_thm1, quot_thm2) andalso eq_option pcr_eq (pcr_info1, pcr_info2) |
53684 | 70 |
|
53754 | 71 |
fun join_restore_data key (rd1:restore_data, rd2) = |
53684 | 72 |
if pointer_eq (rd1, rd2) then raise Symtab.SAME else |
73 |
if not (quotient_eq (#quotient rd1, #quotient rd2)) then raise Symtab.DUP key else |
|
69089 | 74 |
{ quotient = #quotient rd1, |
53684 | 75 |
transfer_rules = Item_Net.merge (#transfer_rules rd1, #transfer_rules rd2)} |
76 |
||
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
77 |
structure Data = Generic_Data |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
78 |
( |
69089 | 79 |
type T = |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
80 |
{ quot_maps : quot_map Symtab.table, |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
81 |
quotients : quotient Symtab.table, |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
82 |
reflexivity_rules : thm Item_Net.T, |
53651 | 83 |
relator_distr_data : relator_distr_data Symtab.table, |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
84 |
restore_data : restore_data Symtab.table, |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
85 |
no_code_types : unit Symtab.table |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
86 |
} |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
87 |
val empty = |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
88 |
{ quot_maps = Symtab.empty, |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
89 |
quotients = Symtab.empty, |
74152 | 90 |
reflexivity_rules = Thm.item_net, |
53651 | 91 |
relator_distr_data = Symtab.empty, |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
92 |
restore_data = Symtab.empty, |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
93 |
no_code_types = Symtab.empty |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
94 |
} |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
95 |
fun merge |
69089 | 96 |
( { quot_maps = qm1, quotients = q1, reflexivity_rules = rr1, relator_distr_data = rdd1, |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
97 |
restore_data = rd1, no_code_types = nct1 }, |
53651 | 98 |
{ quot_maps = qm2, quotients = q2, reflexivity_rules = rr2, relator_distr_data = rdd2, |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
99 |
restore_data = rd2, no_code_types = nct2 } ) = |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
100 |
{ quot_maps = Symtab.merge (K true) (qm1, qm2), |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
101 |
quotients = Symtab.merge (K true) (q1, q2), |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
102 |
reflexivity_rules = Item_Net.merge (rr1, rr2), |
53651 | 103 |
relator_distr_data = Symtab.merge (K true) (rdd1, rdd2), |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
104 |
restore_data = Symtab.join join_restore_data (rd1, rd2), |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
105 |
no_code_types = Symtab.merge (K true) (nct1, nct2) |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
106 |
} |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
107 |
) |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
108 |
|
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
109 |
fun map_data f1 f2 f3 f4 f5 f6 |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
110 |
{ quot_maps, quotients, reflexivity_rules, relator_distr_data, restore_data, no_code_types } = |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
111 |
{ quot_maps = f1 quot_maps, |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
112 |
quotients = f2 quotients, |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
113 |
reflexivity_rules = f3 reflexivity_rules, |
53651 | 114 |
relator_distr_data = f4 relator_distr_data, |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
115 |
restore_data = f5 restore_data, |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
116 |
no_code_types = f6 no_code_types |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
117 |
} |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
118 |
|
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
119 |
fun map_quot_maps f = map_data f I I I I I |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
120 |
fun map_quotients f = map_data I f I I I I |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
121 |
fun map_reflexivity_rules f = map_data I I f I I I |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
122 |
fun map_relator_distr_data f = map_data I I I f I I |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
123 |
fun map_restore_data f = map_data I I I I f I |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
124 |
fun map_no_code_types f = map_data I I I I I f |
69089 | 125 |
|
70320
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
126 |
val get_quot_maps' = #quot_maps o Data.get |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
127 |
val get_quotients' = #quotients o Data.get |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
128 |
val get_reflexivity_rules' = #reflexivity_rules o Data.get |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
129 |
val get_relator_distr_data' = #relator_distr_data o Data.get |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
130 |
val get_restore_data' = #restore_data o Data.get |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
131 |
val get_no_code_types' = #no_code_types o Data.get |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
132 |
|
70320
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
133 |
val get_quot_maps = get_quot_maps' o Context.Proof |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
134 |
val get_quotients = get_quotients' o Context.Proof |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
135 |
val get_relator_distr_data = get_relator_distr_data' o Context.Proof |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
136 |
val get_restore_data = get_restore_data' o Context.Proof |
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
137 |
val get_no_code_types = get_no_code_types' o Context.Proof |
47308 | 138 |
|
69089 | 139 |
|
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
140 |
(* info about Quotient map theorems *) |
47308 | 141 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
142 |
val lookup_quot_maps = Symtab.lookup o get_quot_maps |
47308 | 143 |
|
47784 | 144 |
fun quot_map_thm_sanity_check rel_quot_thm ctxt = |
145 |
let |
|
69089 | 146 |
fun quot_term_absT ctxt quot_term = |
147 |
let |
|
47784 | 148 |
val (_, abs, _, _) = (dest_Quotient o HOLogic.dest_Trueprop) quot_term |
149 |
handle TERM (_, [t]) => error (Pretty.string_of (Pretty.block |
|
150 |
[Pretty.str "The Quotient map theorem is not in the right form.", |
|
151 |
Pretty.brk 1, |
|
152 |
Pretty.str "The following term is not the Quotient predicate:", |
|
153 |
Pretty.brk 1, |
|
154 |
Syntax.pretty_term ctxt t])) |
|
155 |
in |
|
156 |
fastype_of abs |
|
157 |
end |
|
158 |
||
159 |
val ((_, [rel_quot_thm_fixed]), ctxt') = Variable.importT [rel_quot_thm] ctxt |
|
59582 | 160 |
val rel_quot_thm_prop = Thm.prop_of rel_quot_thm_fixed |
47784 | 161 |
val rel_quot_thm_concl = Logic.strip_imp_concl rel_quot_thm_prop |
162 |
val rel_quot_thm_prems = Logic.strip_imp_prems rel_quot_thm_prop; |
|
163 |
val concl_absT = quot_term_absT ctxt' rel_quot_thm_concl |
|
164 |
val concl_tfrees = Term.add_tfree_namesT (concl_absT) [] |
|
69089 | 165 |
val prems_tfrees = fold (fn typ => fn list => Term.add_tfree_namesT (quot_term_absT ctxt' typ) list) |
47784 | 166 |
rel_quot_thm_prems [] |
167 |
val extra_prem_tfrees = |
|
168 |
case subtract (op =) concl_tfrees prems_tfrees of |
|
169 |
[] => [] |
|
170 |
| extras => [Pretty.block ([Pretty.str "Extra type variables in the premises:", |
|
69089 | 171 |
Pretty.brk 1] @ |
47784 | 172 |
((Pretty.commas o map (Pretty.str o quote)) extras) @ |
173 |
[Pretty.str "."])] |
|
69089 | 174 |
val errs = extra_prem_tfrees |
47784 | 175 |
in |
69089 | 176 |
if null errs then () else error (cat_lines (["Sanity check of the quotient map theorem failed:",""] |
47784 | 177 |
@ (map Pretty.string_of errs))) |
178 |
end |
|
179 |
||
180 |
||
69092 | 181 |
fun add_quot_map rel_quot_thm context = |
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
182 |
let |
69092 | 183 |
val _ = Context.cases (K ()) (quot_map_thm_sanity_check rel_quot_thm) context |
59582 | 184 |
val rel_quot_thm_concl = (Logic.strip_imp_concl o Thm.prop_of) rel_quot_thm |
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
185 |
val (_, abs, _, _) = (dest_Quotient o HOLogic.dest_Trueprop) rel_quot_thm_concl |
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
186 |
val relatorT_name = (fst o dest_Type o fst o dest_funT o fastype_of) abs |
70473 | 187 |
val minfo = {rel_quot_thm = Thm.trim_context rel_quot_thm} |
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
188 |
in |
69092 | 189 |
Data.map (map_quot_maps (Symtab.update (relatorT_name, minfo))) context |
69089 | 190 |
end |
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
191 |
|
58821 | 192 |
val _ = |
193 |
Theory.setup |
|
69593 | 194 |
(Attrib.setup \<^binding>\<open>quot_map\<close> (Scan.succeed (Thm.declaration_attribute add_quot_map)) |
58821 | 195 |
"declaration of the Quotient map theorem") |
47308 | 196 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
197 |
fun print_quot_maps ctxt = |
47308 | 198 |
let |
47777
f29e7dcd7c40
use a quot_map theorem attribute instead of the complicated map attribute
kuncar
parents:
47634
diff
changeset
|
199 |
fun prt_map (ty_name, {rel_quot_thm}) = |
47308 | 200 |
Pretty.block (separate (Pretty.brk 2) |
69089 | 201 |
[Pretty.str "type:", |
47308 | 202 |
Pretty.str ty_name, |
69089 | 203 |
Pretty.str "quot. theorem:", |
59582 | 204 |
Syntax.pretty_term ctxt (Thm.prop_of rel_quot_thm)]) |
47308 | 205 |
in |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
206 |
map prt_map (Symtab.dest (get_quot_maps ctxt)) |
47308 | 207 |
|> Pretty.big_list "maps for type constructors:" |
208 |
|> Pretty.writeln |
|
209 |
end |
|
210 |
||
69089 | 211 |
|
47308 | 212 |
(* info about quotient types *) |
53651 | 213 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
214 |
fun transform_pcr_info phi {pcrel_def, pcr_cr_eq} = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
215 |
{pcrel_def = Morphism.thm phi pcrel_def, pcr_cr_eq = Morphism.thm phi pcr_cr_eq} |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
216 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
217 |
fun transform_quotient phi {quot_thm, pcr_info} = |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
218 |
{quot_thm = Morphism.thm phi quot_thm, pcr_info = Option.map (transform_pcr_info phi) pcr_info} |
47308 | 219 |
|
70473 | 220 |
fun lookup_quotients ctxt type_name = |
221 |
Symtab.lookup (get_quotients ctxt) type_name |
|
222 |
|> Option.map (transform_quotient (Morphism.transfer_morphism' ctxt)) |
|
47308 | 223 |
|
60235
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
224 |
fun lookup_quot_thm_quotients ctxt quot_thm = |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
225 |
let |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
226 |
val (_, qtyp) = quot_thm_rty_qty quot_thm |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
227 |
val qty_full_name = (fst o dest_Type) qtyp |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
228 |
fun compare_data (data:quotient) = Thm.eq_thm_prop (#quot_thm data, quot_thm) |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
229 |
in |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
230 |
case lookup_quotients ctxt qty_full_name of |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
231 |
SOME quotient => if compare_data quotient then SOME quotient else NONE |
70320
59258a3192bf
misc tuning and clarification, notably wrt. flow of context;
wenzelm
parents:
69593
diff
changeset
|
232 |
| NONE => NONE |
60235
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
233 |
end |
3cab6f891c2f
reorder some steps in the construction to support mutual datatypes
kuncar
parents:
59936
diff
changeset
|
234 |
|
69092 | 235 |
fun update_quotients type_name qinfo context = |
70473 | 236 |
let val qinfo' = transform_quotient Morphism.trim_context_morphism qinfo |
237 |
in Data.map (map_quotients (Symtab.update (type_name, qinfo'))) context end |
|
47308 | 238 |
|
69092 | 239 |
fun delete_quotients quot_thm context = |
47951
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
240 |
let |
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
241 |
val (_, qtyp) = quot_thm_rty_qty quot_thm |
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
242 |
val qty_full_name = (fst o dest_Type) qtyp |
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
243 |
in |
69092 | 244 |
if is_some (lookup_quot_thm_quotients (Context.proof_of context) quot_thm) |
245 |
then Data.map (map_quotients (Symtab.delete qty_full_name)) context |
|
246 |
else context |
|
47951
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
247 |
end |
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
248 |
|
47308 | 249 |
fun print_quotients ctxt = |
250 |
let |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
251 |
fun prt_quot (qty_name, {quot_thm, pcr_info}: quotient) = |
47308 | 252 |
Pretty.block (separate (Pretty.brk 2) |
70322 | 253 |
([Pretty.str "type:", Pretty.str qty_name, |
254 |
Pretty.str "quot thm:", Thm.pretty_thm ctxt quot_thm] @ |
|
255 |
(case pcr_info of |
|
256 |
NONE => [] |
|
257 |
| SOME {pcrel_def, pcr_cr_eq, ...} => |
|
258 |
[Pretty.str "pcrel_def thm:", Thm.pretty_thm ctxt pcrel_def, |
|
259 |
Pretty.str "pcr_cr_eq thm:", Thm.pretty_thm ctxt pcr_cr_eq]))) |
|
47308 | 260 |
in |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
261 |
map prt_quot (Symtab.dest (get_quotients ctxt)) |
47308 | 262 |
|> Pretty.big_list "quotients:" |
263 |
|> Pretty.writeln |
|
264 |
end |
|
265 |
||
58821 | 266 |
val _ = |
267 |
Theory.setup |
|
69593 | 268 |
(Attrib.setup \<^binding>\<open>quot_del\<close> (Scan.succeed (Thm.declaration_attribute delete_quotients)) |
58821 | 269 |
"deletes the Quotient theorem") |
47951
8c8a03765de7
quot_del attribute, it allows us to deregister quotient types
kuncar
parents:
47936
diff
changeset
|
270 |
|
53651 | 271 |
(* data for restoring Transfer/Lifting context *) |
272 |
||
273 |
fun lookup_restore_data ctxt bundle_name = Symtab.lookup (get_restore_data ctxt) bundle_name |
|
274 |
||
69092 | 275 |
fun update_restore_data bundle_name restore_data context = |
276 |
Data.map (map_restore_data (Symtab.update (bundle_name, restore_data))) context |
|
53651 | 277 |
|
69092 | 278 |
fun init_restore_data bundle_name qinfo context = |
74152 | 279 |
update_restore_data bundle_name { quotient = qinfo, transfer_rules = Thm.item_net } context |
53651 | 280 |
|
69092 | 281 |
fun add_transfer_rules_in_restore_data bundle_name transfer_rules context = |
282 |
(case Symtab.lookup (get_restore_data' context) bundle_name of |
|
283 |
SOME restore_data => |
|
284 |
update_restore_data bundle_name { quotient = #quotient restore_data, |
|
285 |
transfer_rules = Item_Net.merge ((#transfer_rules restore_data), transfer_rules) } context |
|
286 |
| NONE => error ("The restore data " ^ quote bundle_name ^ " is not defined.")) |
|
53651 | 287 |
|
69089 | 288 |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
289 |
(* theorems that a relator of an eq_onp is an eq_onp of the corresponding predicate *) |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
290 |
|
57961 | 291 |
fun get_relator_eq_onp_rules ctxt = |
69593 | 292 |
map safe_mk_meta_eq (rev (Named_Theorems.get ctxt \<^named_theorems>\<open>relator_eq_onp\<close>)) |
47634
091bcd569441
hide the invariant constant for relators: invariant_commute infrastracture
kuncar
parents:
47308
diff
changeset
|
293 |
|
69089 | 294 |
|
51994 | 295 |
(* info about reflexivity rules *) |
296 |
||
70473 | 297 |
fun get_reflexivity_rules ctxt = |
298 |
Item_Net.content (get_reflexivity_rules' (Context.Proof ctxt)) |
|
299 |
|> map (Thm.transfer' ctxt) |
|
51994 | 300 |
|
70473 | 301 |
fun add_reflexivity_rule thm = |
302 |
Data.map (map_reflexivity_rules (Item_Net.update (Thm.trim_context thm))) |
|
303 |
||
51994 | 304 |
val add_reflexivity_rule_attribute = Thm.declaration_attribute add_reflexivity_rule |
305 |
||
69089 | 306 |
|
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
307 |
(* info about relator distributivity theorems *) |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
308 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
309 |
fun map_relator_distr_data' f1 f2 f3 f4 |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
310 |
{pos_mono_rule, neg_mono_rule, pos_distr_rules, neg_distr_rules} = |
69089 | 311 |
{pos_mono_rule = f1 pos_mono_rule, |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
312 |
neg_mono_rule = f2 neg_mono_rule, |
69089 | 313 |
pos_distr_rules = f3 pos_distr_rules, |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
314 |
neg_distr_rules = f4 neg_distr_rules} |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
315 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
316 |
fun map_pos_mono_rule f = map_relator_distr_data' f I I I |
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
317 |
fun map_neg_mono_rule f = map_relator_distr_data' I f I I |
69089 | 318 |
fun map_pos_distr_rules f = map_relator_distr_data' I I f I |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
319 |
fun map_neg_distr_rules f = map_relator_distr_data' I I I f |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
320 |
|
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
321 |
fun introduce_polarities rule = |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
322 |
let |
69593 | 323 |
val dest_less_eq = HOLogic.dest_bin \<^const_name>\<open>less_eq\<close> dummyT |
59582 | 324 |
val prems_pairs = map (dest_less_eq o HOLogic.dest_Trueprop) (Thm.prems_of rule) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
325 |
val equal_prems = filter op= prems_pairs |
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58893
diff
changeset
|
326 |
val _ = |
69089 | 327 |
if null equal_prems then () |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
328 |
else error "The rule contains reflexive assumptions." |
69089 | 329 |
val concl_pairs = rule |
59582 | 330 |
|> Thm.concl_of |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
331 |
|> HOLogic.dest_Trueprop |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
332 |
|> dest_less_eq |
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58893
diff
changeset
|
333 |
|> apply2 (snd o strip_comb) |
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58893
diff
changeset
|
334 |
|> op ~~ |
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58893
diff
changeset
|
335 |
|> filter_out op = |
69089 | 336 |
|
337 |
val _ = if has_duplicates op= concl_pairs |
|
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
338 |
then error "The rule contains duplicated variables in the conlusion." else () |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
339 |
|
69089 | 340 |
fun rewrite_prem prem_pair = |
51427
08bb00239652
proper use of "member", without embarking on delicate questions about SML equality types;
wenzelm
parents:
51426
diff
changeset
|
341 |
if member op= concl_pairs prem_pair |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
342 |
then HOLogic.Trueprop_conv (Conv.rewr_conv (Thm.symmetric @{thm POS_def})) |
51427
08bb00239652
proper use of "member", without embarking on delicate questions about SML equality types;
wenzelm
parents:
51426
diff
changeset
|
343 |
else if member op= concl_pairs (swap prem_pair) |
59058
a78612c67ec0
renamed "pairself" to "apply2", in accordance to @{apply 2};
wenzelm
parents:
58893
diff
changeset
|
344 |
then HOLogic.Trueprop_conv (Conv.rewr_conv (Thm.symmetric @{thm NEG_def})) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
345 |
else error "The rule contains a non-relevant assumption." |
69089 | 346 |
|
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
347 |
fun rewrite_prems [] = Conv.all_conv |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
348 |
| rewrite_prems (x::xs) = Conv.implies_conv (rewrite_prem x) (rewrite_prems xs) |
69089 | 349 |
|
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
350 |
val rewrite_prems_conv = rewrite_prems prems_pairs |
69089 | 351 |
val rewrite_concl_conv = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
352 |
Conv.concl_conv ~1 (HOLogic.Trueprop_conv (Conv.rewr_conv (Thm.symmetric @{thm POS_def}))) |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
353 |
in |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
354 |
(Conv.fconv_rule (rewrite_prems_conv then_conv rewrite_concl_conv)) rule |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
355 |
end |
69089 | 356 |
handle |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
357 |
TERM _ => error "The rule has a wrong format." |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
358 |
| CTERM _ => error "The rule has a wrong format." |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
359 |
|
69089 | 360 |
fun negate_mono_rule mono_rule = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
361 |
let |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
362 |
val rewr_conv = HOLogic.Trueprop_conv (Conv.rewrs_conv [@{thm POS_NEG}, @{thm NEG_POS}]) |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
363 |
in |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
364 |
Conv.fconv_rule (Conv.prems_conv ~1 rewr_conv then_conv Conv.concl_conv ~1 rewr_conv) mono_rule |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
365 |
end; |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
366 |
|
69092 | 367 |
fun add_reflexivity_rules mono_rule context = |
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
368 |
let |
70473 | 369 |
val ctxt = Context.proof_of context |
370 |
val thy = Context.theory_of context |
|
371 |
||
372 |
fun find_eq_rule thm = |
|
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
373 |
let |
70473 | 374 |
val concl_rhs = (hd o get_args 1 o HOLogic.dest_Trueprop o Thm.concl_of) thm |
375 |
val rules = Transfer.retrieve_relator_eq ctxt concl_rhs |
|
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
376 |
in |
70473 | 377 |
find_first (fn th => Pattern.matches thy (concl_rhs, |
378 |
(fst o HOLogic.dest_eq o HOLogic.dest_Trueprop o Thm.concl_of) th)) rules |
|
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
379 |
end |
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
380 |
|
70473 | 381 |
val eq_rule = find_eq_rule mono_rule; |
69089 | 382 |
val eq_rule = if is_some eq_rule then the eq_rule else error |
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
383 |
"No corresponding rule that the relator preserves equality was found." |
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
384 |
in |
69092 | 385 |
context |
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
386 |
|> add_reflexivity_rule (Drule.zero_var_indexes (@{thm ord_le_eq_trans} OF [mono_rule, eq_rule])) |
69089 | 387 |
|> add_reflexivity_rule |
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
388 |
(Drule.zero_var_indexes (@{thm ord_eq_le_trans} OF [sym OF [eq_rule], mono_rule])) |
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
389 |
end |
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
390 |
|
69092 | 391 |
fun add_mono_rule mono_rule context = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
392 |
let |
55563
a64d49f49ca3
implement the reflexivity prover as a monotonicity prover that proves R >= op=; derive "reflexivity" rules for relators from mono rules and eq rules
kuncar
parents:
53754
diff
changeset
|
393 |
val pol_mono_rule = introduce_polarities mono_rule |
69089 | 394 |
val mono_ruleT_name = (fst o dest_Type o fst o relation_types o fst o relation_types o snd o |
59582 | 395 |
dest_Const o head_of o HOLogic.dest_Trueprop o Thm.concl_of) pol_mono_rule |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
396 |
in |
69092 | 397 |
if Symtab.defined (get_relator_distr_data' context) mono_ruleT_name |
69091
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
398 |
then |
69092 | 399 |
(if Context_Position.is_visible_generic context then |
69091
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
400 |
warning ("Monotonicity rule for type " ^ quote mono_ruleT_name ^ " is already_defined.") |
69092 | 401 |
else (); context) |
69091
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
402 |
else |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
403 |
let |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
404 |
val neg_mono_rule = negate_mono_rule pol_mono_rule |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
405 |
val relator_distr_data = {pos_mono_rule = pol_mono_rule, neg_mono_rule = neg_mono_rule, |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
406 |
pos_distr_rules = [], neg_distr_rules = []} |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
407 |
in |
69092 | 408 |
context |
69091
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
409 |
|> Data.map (map_relator_distr_data (Symtab.update (mono_ruleT_name, relator_distr_data))) |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
410 |
|> add_reflexivity_rules mono_rule |
ce62fd14961a
permissive declaration attribute "relator_mono", e.g. relevant for Binomial-Heaps.BinomialHeap with -o export_theory;
wenzelm
parents:
69090
diff
changeset
|
411 |
end |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
412 |
end; |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
413 |
|
69089 | 414 |
local |
69092 | 415 |
fun add_distr_rule update_entry distr_rule context = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
416 |
let |
69089 | 417 |
val distr_ruleT_name = (fst o dest_Type o fst o relation_types o fst o relation_types o snd o |
59582 | 418 |
dest_Const o head_of o HOLogic.dest_Trueprop o Thm.concl_of) distr_rule |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
419 |
in |
69092 | 420 |
if Symtab.defined (get_relator_distr_data' context) distr_ruleT_name then |
69089 | 421 |
Data.map (map_relator_distr_data (Symtab.map_entry distr_ruleT_name (update_entry distr_rule))) |
69092 | 422 |
context |
69090 | 423 |
else error "The monotonicity rule is not defined." |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
424 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
425 |
|
69090 | 426 |
fun rewrite_concl_conv thm ctm = |
427 |
Conv.concl_conv ~1 (HOLogic.Trueprop_conv (Conv.rewr_conv (Thm.symmetric thm))) ctm |
|
428 |
handle CTERM _ => error "The rule has a wrong format." |
|
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
429 |
|
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
430 |
in |
69092 | 431 |
fun add_pos_distr_rule distr_rule context = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
432 |
let |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
433 |
val distr_rule = Conv.fconv_rule (rewrite_concl_conv @{thm POS_def}) distr_rule |
69089 | 434 |
fun update_entry distr_rule data = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
435 |
map_pos_distr_rules (cons (@{thm POS_trans} OF [distr_rule, #pos_mono_rule data])) data |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
436 |
in |
69092 | 437 |
add_distr_rule update_entry distr_rule context |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
438 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
439 |
handle THM _ => error "Combining of the distr. rule and the monotonicity rule together has failed." |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
440 |
|
69092 | 441 |
fun add_neg_distr_rule distr_rule context = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
442 |
let |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
443 |
val distr_rule = Conv.fconv_rule (rewrite_concl_conv @{thm NEG_def}) distr_rule |
69089 | 444 |
fun update_entry distr_rule data = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
445 |
map_neg_distr_rules (cons (@{thm NEG_trans} OF [distr_rule, #neg_mono_rule data])) data |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
446 |
in |
69092 | 447 |
add_distr_rule update_entry distr_rule context |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
448 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
449 |
handle THM _ => error "Combining of the distr. rule and the monotonicity rule together has failed." |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
450 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
451 |
|
69089 | 452 |
local |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
453 |
val eq_refl2 = sym RS @{thm eq_refl} |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
454 |
in |
69092 | 455 |
fun add_eq_distr_rule distr_rule context = |
69089 | 456 |
let |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
457 |
val pos_distr_rule = @{thm eq_refl} OF [distr_rule] |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
458 |
val neg_distr_rule = eq_refl2 OF [distr_rule] |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
459 |
in |
69092 | 460 |
context |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
461 |
|> add_pos_distr_rule pos_distr_rule |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
462 |
|> add_neg_distr_rule neg_distr_rule |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
463 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
464 |
end; |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
465 |
|
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
466 |
local |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
467 |
fun sanity_check rule = |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
468 |
let |
59582 | 469 |
val assms = map (perhaps (try HOLogic.dest_Trueprop)) (Thm.prems_of rule) |
470 |
val concl = (perhaps (try HOLogic.dest_Trueprop)) (Thm.concl_of rule); |
|
56257 | 471 |
val (lhs, rhs) = |
472 |
(case concl of |
|
69593 | 473 |
Const (\<^const_name>\<open>less_eq\<close>, _) $ (lhs as Const (\<^const_name>\<open>relcompp\<close>,_) $ _ $ _) $ rhs => |
56257 | 474 |
(lhs, rhs) |
69593 | 475 |
| Const (\<^const_name>\<open>less_eq\<close>, _) $ rhs $ (lhs as Const (\<^const_name>\<open>relcompp\<close>,_) $ _ $ _) => |
56257 | 476 |
(lhs, rhs) |
69593 | 477 |
| Const (\<^const_name>\<open>HOL.eq\<close>, _) $ (lhs as Const (\<^const_name>\<open>relcompp\<close>,_) $ _ $ _) $ rhs => |
56257 | 478 |
(lhs, rhs) |
479 |
| _ => error "The rule has a wrong format.") |
|
69089 | 480 |
|
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
481 |
val lhs_vars = Term.add_vars lhs [] |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
482 |
val rhs_vars = Term.add_vars rhs [] |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
483 |
val assms_vars = fold Term.add_vars assms []; |
56257 | 484 |
val _ = |
485 |
if has_duplicates op= lhs_vars |
|
486 |
then error "Left-hand side has variable duplicates" else () |
|
487 |
val _ = |
|
69089 | 488 |
if subset op= (rhs_vars, lhs_vars) then () |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
489 |
else error "Extra variables in the right-hand side of the rule" |
56257 | 490 |
val _ = |
69089 | 491 |
if subset op= (assms_vars, lhs_vars) then () |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
492 |
else error "Extra variables in the assumptions of the rule" |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
493 |
val rhs_args = (snd o strip_comb) rhs; |
56257 | 494 |
fun check_comp t = |
495 |
(case t of |
|
69593 | 496 |
Const (\<^const_name>\<open>relcompp\<close>, _) $ Var _ $ Var _ => () |
56257 | 497 |
| _ => error "There is an argument on the rhs that is not a composition.") |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
498 |
val _ = map check_comp rhs_args |
56257 | 499 |
in () end |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
500 |
in |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
501 |
|
69092 | 502 |
fun add_distr_rule distr_rule context = |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
503 |
let |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
504 |
val _ = sanity_check distr_rule |
59582 | 505 |
val concl = (perhaps (try HOLogic.dest_Trueprop)) (Thm.concl_of distr_rule) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
506 |
in |
56257 | 507 |
(case concl of |
69593 | 508 |
Const (\<^const_name>\<open>less_eq\<close>, _) $ (Const (\<^const_name>\<open>relcompp\<close>,_) $ _ $ _) $ _ => |
69092 | 509 |
add_pos_distr_rule distr_rule context |
69593 | 510 |
| Const (\<^const_name>\<open>less_eq\<close>, _) $ _ $ (Const (\<^const_name>\<open>relcompp\<close>,_) $ _ $ _) => |
69092 | 511 |
add_neg_distr_rule distr_rule context |
69593 | 512 |
| Const (\<^const_name>\<open>HOL.eq\<close>, _) $ (Const (\<^const_name>\<open>relcompp\<close>,_) $ _ $ _) $ _ => |
69092 | 513 |
add_eq_distr_rule distr_rule context) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
514 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
515 |
end |
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
516 |
|
70473 | 517 |
fun get_distr_rules_raw context = |
518 |
Symtab.fold (fn (_, {pos_distr_rules, neg_distr_rules, ...}) => fn rules => |
|
519 |
pos_distr_rules @ neg_distr_rules @ rules) |
|
69092 | 520 |
(get_relator_distr_data' context) [] |
70473 | 521 |
|> map (Thm.transfer'' context) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
522 |
|
70473 | 523 |
fun get_mono_rules_raw context = |
524 |
Symtab.fold (fn (_, {pos_mono_rule, neg_mono_rule, ...}) => fn rules => |
|
525 |
[pos_mono_rule, neg_mono_rule] @ rules) |
|
69092 | 526 |
(get_relator_distr_data' context) [] |
70473 | 527 |
|> map (Thm.transfer'' context) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
528 |
|
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
529 |
val lookup_relator_distr_data = Symtab.lookup o get_relator_distr_data |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
530 |
|
58821 | 531 |
val _ = |
532 |
Theory.setup |
|
69593 | 533 |
(Attrib.setup \<^binding>\<open>relator_mono\<close> (Scan.succeed (Thm.declaration_attribute add_mono_rule)) |
69090 | 534 |
"declaration of relator's monotonicity" |
69593 | 535 |
#> Attrib.setup \<^binding>\<open>relator_distr\<close> (Scan.succeed (Thm.declaration_attribute add_distr_rule)) |
58821 | 536 |
"declaration of relator's distributivity over OO" |
537 |
#> Global_Theory.add_thms_dynamic |
|
69593 | 538 |
(\<^binding>\<open>relator_distr_raw\<close>, get_distr_rules_raw) |
58821 | 539 |
#> Global_Theory.add_thms_dynamic |
69593 | 540 |
(\<^binding>\<open>relator_mono_raw\<close>, get_mono_rules_raw)) |
51374
84d01fd733cf
lift_definition and setup_lifting generate parametric transfer rules if parametricity theorems are provided
kuncar
parents:
50227
diff
changeset
|
541 |
|
69089 | 542 |
|
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
543 |
(* no_code types *) |
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
544 |
|
69092 | 545 |
fun add_no_code_type type_name context = |
546 |
Data.map (map_no_code_types (Symtab.update (type_name, ()))) context; |
|
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
547 |
|
69092 | 548 |
fun is_no_code_type context type_name = (Symtab.defined o get_no_code_types) context type_name |
57663
b590fcd03a4a
store explicitly quotient types with no_code => more precise registration of code equations
kuncar
parents:
56519
diff
changeset
|
549 |
|
69089 | 550 |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
551 |
(* setup fixed eq_onp rules *) |
55731
66df76dd2640
rewrite composition of quotients to a more readable form in a respectfulness goal that is presented to a user
kuncar
parents:
55563
diff
changeset
|
552 |
|
57961 | 553 |
val _ = Context.>> |
69593 | 554 |
(fold (Named_Theorems.add_thm \<^named_theorems>\<open>relator_eq_onp\<close> o |
555 |
Transfer.prep_transfer_domain_thm \<^context>) |
|
56519
c1048f5bbb45
more appropriate name (Lifting.invariant -> eq_onp)
kuncar
parents:
56518
diff
changeset
|
556 |
@{thms composed_equiv_rel_eq_onp composed_equiv_rel_eq_eq_onp}) |
56518
beb3b6851665
left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
kuncar
parents:
56257
diff
changeset
|
557 |
|
69089 | 558 |
|
56518
beb3b6851665
left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
kuncar
parents:
56257
diff
changeset
|
559 |
(* setup fixed reflexivity rules *) |
beb3b6851665
left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
kuncar
parents:
56257
diff
changeset
|
560 |
|
69089 | 561 |
val _ = Context.>> (fold add_reflexivity_rule |
67399 | 562 |
@{thms order_refl[of "(=)"] eq_onp_le_eq Quotient_composition_le_eq Quotient_composition_ge_eq |
56518
beb3b6851665
left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
kuncar
parents:
56257
diff
changeset
|
563 |
bi_unique_OO bi_total_OO right_unique_OO right_total_OO left_unique_OO left_total_OO}) |
55731
66df76dd2640
rewrite composition of quotients to a more readable form in a respectfulness goal that is presented to a user
kuncar
parents:
55563
diff
changeset
|
564 |
|
69089 | 565 |
|
47308 | 566 |
(* outer syntax commands *) |
567 |
||
568 |
val _ = |
|
69593 | 569 |
Outer_Syntax.command \<^command_keyword>\<open>print_quot_maps\<close> "print quotient map functions" |
53219
ca237b9e4542
use only one data slot; rename print_quotmaps to print_quot_maps; tuned
kuncar
parents:
51994
diff
changeset
|
570 |
(Scan.succeed (Toplevel.keep (print_quot_maps o Toplevel.context_of))) |
47308 | 571 |
|
572 |
val _ = |
|
69593 | 573 |
Outer_Syntax.command \<^command_keyword>\<open>print_quotients\<close> "print quotients" |
47308 | 574 |
(Scan.succeed (Toplevel.keep (print_quotients o Toplevel.context_of))) |
575 |
||
53651 | 576 |
end |