author | Christian Urban <urbanc@in.tum.de> |
Mon, 16 Jan 2012 12:42:47 +0000 | |
changeset 3108 | 61db5ad429bb |
parent 3045 | d0ad264f8c4f |
child 3197 | 25d11b449e92 |
permissions | -rw-r--r-- |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1 |
(* Nominal Function Core |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
2 |
Author: Christian Urban |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
3 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
4 |
heavily based on the code of Alexander Krauss |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
5 |
(code forked on 14 January 2011) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
6 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
7 |
Core of the nominal function package. |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
8 |
*) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
9 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
10 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
11 |
signature NOMINAL_FUNCTION_CORE = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
12 |
sig |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
13 |
val trace: bool Unsynchronized.ref |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
14 |
|
2819
4bd584ff4fab
added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents:
2803
diff
changeset
|
15 |
val prepare_nominal_function : Nominal_Function_Common.nominal_function_config |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
16 |
-> string (* defname *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
17 |
-> ((bstring * typ) * mixfix) list (* defined symbol *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
18 |
-> ((bstring * typ) list * term list * term * term) list (* specification *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
19 |
-> local_theory |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
20 |
-> (term (* f *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
21 |
* thm (* goalstate *) |
2973
d1038e67923a
added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents:
2885
diff
changeset
|
22 |
* (thm -> Nominal_Function_Common.nominal_function_result) (* continuation *) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
23 |
) * local_theory |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
24 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
25 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
26 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
27 |
structure Nominal_Function_Core : NOMINAL_FUNCTION_CORE = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
28 |
struct |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
29 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
30 |
val trace = Unsynchronized.ref false |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
31 |
fun trace_msg msg = if ! trace then tracing (msg ()) else () |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
32 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
33 |
val boolT = HOLogic.boolT |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
34 |
val mk_eq = HOLogic.mk_eq |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
35 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
36 |
open Function_Lib |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
37 |
open Function_Common |
2819
4bd584ff4fab
added an option for an invariant (at the moment only a stub)
Christian Urban <urbanc@in.tum.de>
parents:
2803
diff
changeset
|
38 |
open Nominal_Function_Common |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
39 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
40 |
datatype globals = Globals of |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
41 |
{fvar: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
42 |
domT: typ, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
43 |
ranT: typ, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
44 |
h: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
45 |
y: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
46 |
x: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
47 |
z: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
48 |
a: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
49 |
P: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
50 |
D: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
51 |
Pbool:term} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
52 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
53 |
datatype rec_call_info = RCInfo of |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
54 |
{RIvs: (string * typ) list, (* Call context: fixes and assumes *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
55 |
CCas: thm list, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
56 |
rcarg: term, (* The recursive argument *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
57 |
llRI: thm, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
58 |
h_assum: term} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
59 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
60 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
61 |
datatype clause_context = ClauseContext of |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
62 |
{ctxt : Proof.context, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
63 |
qs : term list, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
64 |
gs : term list, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
65 |
lhs: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
66 |
rhs: term, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
67 |
cqs: cterm list, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
68 |
ags: thm list, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
69 |
case_hyp : thm} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
70 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
71 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
72 |
fun transfer_clause_ctx thy (ClauseContext { ctxt, qs, gs, lhs, rhs, cqs, ags, case_hyp }) = |
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
73 |
ClauseContext { ctxt = Proof_Context.transfer thy ctxt, |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
74 |
qs = qs, gs = gs, lhs = lhs, rhs = rhs, cqs = cqs, ags = ags, case_hyp = case_hyp } |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
75 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
76 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
77 |
datatype clause_info = ClauseInfo of |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
78 |
{no: int, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
79 |
qglr : ((string * typ) list * term list * term * term), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
80 |
cdata : clause_context, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
81 |
tree: Function_Ctx_Tree.ctx_tree, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
82 |
lGI: thm, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
83 |
RCs: rec_call_info list} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
84 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
85 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
86 |
(* Theory dependencies. *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
87 |
val acc_induct_rule = @{thm accp_induct_rule} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
88 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
89 |
val ex1_implies_ex = @{thm FunDef.fundef_ex1_existence} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
90 |
val ex1_implies_un = @{thm FunDef.fundef_ex1_uniqueness} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
91 |
val ex1_implies_iff = @{thm FunDef.fundef_ex1_iff} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
92 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
93 |
val acc_downward = @{thm accp_downward} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
94 |
val accI = @{thm accp.accI} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
95 |
val case_split = @{thm HOL.case_split} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
96 |
val fundef_default_value = @{thm FunDef.fundef_default_value} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
97 |
val not_acc_down = @{thm not_accp_down} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
98 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
99 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
100 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
101 |
fun find_calls tree = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
102 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
103 |
fun add_Ri (fixes,assumes) (_ $ arg) _ (_, xs) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
104 |
([], (fixes, assumes, arg) :: xs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
105 |
| add_Ri _ _ _ _ = raise Match |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
106 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
107 |
rev (Function_Ctx_Tree.traverse_tree add_Ri tree []) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
108 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
109 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
110 |
(* nominal *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
111 |
fun mk_eqvt_at (f_trm, arg_trm) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
112 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
113 |
val f_ty = fastype_of f_trm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
114 |
val arg_ty = domain_type f_ty |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
115 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
116 |
Const (@{const_name eqvt_at}, [f_ty, arg_ty] ---> @{typ bool}) $ f_trm $ arg_trm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
117 |
|> HOLogic.mk_Trueprop |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
118 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
119 |
|
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
120 |
fun mk_eqvt trm = |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
121 |
let |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
122 |
val ty = fastype_of trm |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
123 |
in |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
124 |
Const (@{const_name eqvt}, ty --> @{typ bool}) $ trm |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
125 |
|> HOLogic.mk_Trueprop |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
126 |
end |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
127 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
128 |
fun mk_inv inv (f_trm, arg_trm) = |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
129 |
betapplys (inv, [arg_trm, (f_trm $ arg_trm)]) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
130 |
|> HOLogic.mk_Trueprop |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
131 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
132 |
fun mk_invariant (Globals {x, y, ...}) G invariant = |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
133 |
let |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
134 |
val prem = HOLogic.mk_Trueprop (G $ x $ y) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
135 |
val concl = HOLogic.mk_Trueprop (betapplys (invariant, [x, y])) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
136 |
in |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
137 |
Logic.mk_implies (prem, concl) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
138 |
|> mk_forall_rename ("y", y) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
139 |
|> mk_forall_rename ("x", x) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
140 |
end |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
141 |
|
2790 | 142 |
(** building proof obligations *) |
2802
3b9ef98a03d2
first test to fix the problem with free variables
Christian Urban <urbanc@in.tum.de>
parents:
2796
diff
changeset
|
143 |
fun mk_eqvt_proof_obligation qs fvar (vs, assms, arg) = |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
144 |
mk_eqvt_at (fvar, arg) |
2803
04f7c4ce8588
hopefully final fix for ho-functions
Christian Urban <urbanc@in.tum.de>
parents:
2802
diff
changeset
|
145 |
|> curry Logic.list_implies (map prop_of assms) |
3108
61db5ad429bb
updated to Isabelle 16 January
Christian Urban <urbanc@in.tum.de>
parents:
3045
diff
changeset
|
146 |
|> fold_rev (Logic.all o Free) vs |
2994
4ee772b12032
Update to new Isabelle
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
2974
diff
changeset
|
147 |
|> fold_rev absfree qs |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
148 |
|> strip_abs_body |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
149 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
150 |
fun mk_inv_proof_obligation inv qs fvar (vs, assms, arg) = |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
151 |
mk_inv inv (fvar, arg) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
152 |
|> curry Logic.list_implies (map prop_of assms) |
3108
61db5ad429bb
updated to Isabelle 16 January
Christian Urban <urbanc@in.tum.de>
parents:
3045
diff
changeset
|
153 |
|> fold_rev (Logic.all o Free) vs |
2994
4ee772b12032
Update to new Isabelle
Cezary Kaliszyk <kaliszyk@in.tum.de>
parents:
2974
diff
changeset
|
154 |
|> fold_rev absfree qs |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
155 |
|> strip_abs_body |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
156 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
157 |
(** building proof obligations *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
158 |
fun mk_compat_proof_obligations domT ranT fvar f RCss inv glrs = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
159 |
let |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
160 |
fun mk_impl (((qs, gs, lhs, rhs), RCs_lhs), ((qs', gs', lhs', rhs'), RCs_rhs)) = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
161 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
162 |
val shift = incr_boundvars (length qs') |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
163 |
val eqvts_obligations_lhs = map (shift o mk_eqvt_proof_obligation qs fvar) RCs_lhs |
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
164 |
val eqvts_obligations_rhs = map (mk_eqvt_proof_obligation qs' fvar) RCs_rhs |
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
165 |
val invs_obligations_lhs = map (shift o mk_inv_proof_obligation inv qs fvar) RCs_lhs |
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
166 |
val invs_obligations_rhs = map (mk_inv_proof_obligation inv qs' fvar) RCs_rhs |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
167 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
168 |
Logic.mk_implies |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
169 |
(HOLogic.mk_Trueprop (HOLogic.eq_const domT $ shift lhs $ lhs'), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
170 |
HOLogic.mk_Trueprop (HOLogic.eq_const ranT $ shift rhs $ rhs')) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
171 |
|> fold_rev (curry Logic.mk_implies) (map shift gs @ gs') |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
172 |
|> fold_rev (curry Logic.mk_implies) invs_obligations_rhs (* nominal *) |
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
173 |
|> fold_rev (curry Logic.mk_implies) invs_obligations_lhs (* nominal *) |
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
174 |
|> fold_rev (curry Logic.mk_implies) eqvts_obligations_rhs (* nominal *) |
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
175 |
|> fold_rev (curry Logic.mk_implies) eqvts_obligations_lhs (* nominal *) |
3108
61db5ad429bb
updated to Isabelle 16 January
Christian Urban <urbanc@in.tum.de>
parents:
3045
diff
changeset
|
176 |
|> fold_rev (fn (n,T) => fn b => Logic.all_const T $ Abs(n,T,b)) (qs @ qs') |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
177 |
|> curry abstract_over fvar |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
178 |
|> curry subst_bound f |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
179 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
180 |
in |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
181 |
map mk_impl (unordered_pairs (glrs ~~ RCss)) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
182 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
183 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
184 |
fun mk_completeness (Globals {x, Pbool, ...}) clauses qglrs = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
185 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
186 |
fun mk_case (ClauseContext {qs, gs, lhs, ...}, (oqs, _, _, _)) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
187 |
HOLogic.mk_Trueprop Pbool |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
188 |
|> curry Logic.mk_implies (HOLogic.mk_Trueprop (mk_eq (x, lhs))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
189 |
|> fold_rev (curry Logic.mk_implies) gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
190 |
|> fold_rev mk_forall_rename (map fst oqs ~~ qs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
191 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
192 |
HOLogic.mk_Trueprop Pbool |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
193 |
|> fold_rev (curry Logic.mk_implies o mk_case) (clauses ~~ qglrs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
194 |
|> mk_forall_rename ("x", x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
195 |
|> mk_forall_rename ("P", Pbool) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
196 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
197 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
198 |
(** making a context with it's own local bindings **) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
199 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
200 |
fun mk_clause_context x ctxt (pre_qs,pre_gs,pre_lhs,pre_rhs) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
201 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
202 |
val (qs, ctxt') = Variable.variant_fixes (map fst pre_qs) ctxt |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
203 |
|>> map2 (fn (_, T) => fn n => Free (n, T)) pre_qs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
204 |
|
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
205 |
val thy = Proof_Context.theory_of ctxt' |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
206 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
207 |
fun inst t = subst_bounds (rev qs, t) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
208 |
val gs = map inst pre_gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
209 |
val lhs = inst pre_lhs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
210 |
val rhs = inst pre_rhs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
211 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
212 |
val cqs = map (cterm_of thy) qs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
213 |
val ags = map (Thm.assume o cterm_of thy) gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
214 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
215 |
val case_hyp = Thm.assume (cterm_of thy (HOLogic.mk_Trueprop (mk_eq (x, lhs)))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
216 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
217 |
ClauseContext { ctxt = ctxt', qs = qs, gs = gs, lhs = lhs, rhs = rhs, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
218 |
cqs = cqs, ags = ags, case_hyp = case_hyp } |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
219 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
220 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
221 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
222 |
(* lowlevel term function. FIXME: remove *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
223 |
fun abstract_over_list vs body = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
224 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
225 |
fun abs lev v tm = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
226 |
if v aconv tm then Bound lev |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
227 |
else |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
228 |
(case tm of |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
229 |
Abs (a, T, t) => Abs (a, T, abs (lev + 1) v t) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
230 |
| t $ u => abs lev v t $ abs lev v u |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
231 |
| t => t) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
232 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
233 |
fold_index (fn (i, v) => fn t => abs i v t) vs body |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
234 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
235 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
236 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
237 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
238 |
fun mk_clause_info globals G f no cdata qglr tree RCs GIntro_thm RIntro_thms = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
239 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
240 |
val Globals {h, ...} = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
241 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
242 |
val ClauseContext { ctxt, qs, cqs, ags, ... } = cdata |
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
243 |
val cert = Thm.cterm_of (Proof_Context.theory_of ctxt) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
244 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
245 |
(* Instantiate the GIntro thm with "f" and import into the clause context. *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
246 |
val lGI = GIntro_thm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
247 |
|> Thm.forall_elim (cert f) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
248 |
|> fold Thm.forall_elim cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
249 |
|> fold Thm.elim_implies ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
250 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
251 |
fun mk_call_info (rcfix, rcassm, rcarg) RI = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
252 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
253 |
val llRI = RI |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
254 |
|> fold Thm.forall_elim cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
255 |
|> fold (Thm.forall_elim o cert o Free) rcfix |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
256 |
|> fold Thm.elim_implies ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
257 |
|> fold Thm.elim_implies rcassm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
258 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
259 |
val h_assum = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
260 |
HOLogic.mk_Trueprop (G $ rcarg $ (h $ rcarg)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
261 |
|> fold_rev (curry Logic.mk_implies o prop_of) rcassm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
262 |
|> fold_rev (Logic.all o Free) rcfix |
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
263 |
|> Pattern.rewrite_term (Proof_Context.theory_of ctxt) [(f, h)] [] |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
264 |
|> abstract_over_list (rev qs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
265 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
266 |
RCInfo {RIvs=rcfix, rcarg=rcarg, CCas=rcassm, llRI=llRI, h_assum=h_assum} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
267 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
268 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
269 |
val RC_infos = map2 mk_call_info RCs RIntro_thms |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
270 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
271 |
ClauseInfo {no=no, cdata=cdata, qglr=qglr, lGI=lGI, RCs=RC_infos, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
272 |
tree=tree} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
273 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
274 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
275 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
276 |
fun store_compat_thms 0 thms = [] |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
277 |
| store_compat_thms n thms = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
278 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
279 |
val (thms1, thms2) = chop n thms |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
280 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
281 |
(thms1 :: store_compat_thms (n - 1) thms2) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
282 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
283 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
284 |
(* expects i <= j *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
285 |
fun lookup_compat_thm i j cts = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
286 |
nth (nth cts (i - 1)) (j - i) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
287 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
288 |
(* nominal *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
289 |
(* Returns "Gsi, Gsj, lhs_i = lhs_j |-- rhs_j_f = rhs_i_f" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
290 |
(* if j < i, then turn around *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
291 |
fun get_compat_thm thy cts eqvtsi eqvtsj invsi invsj i j ctxi ctxj = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
292 |
let |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
293 |
val ClauseContext {cqs=cqsi,ags=agsi,lhs=lhsi,case_hyp=case_hypi,...} = ctxi |
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
294 |
val ClauseContext {cqs=cqsj,ags=agsj,lhs=lhsj,case_hyp=case_hypj,...} = ctxj |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
295 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
296 |
val lhsi_eq_lhsj = cterm_of thy (HOLogic.mk_Trueprop (mk_eq (lhsi, lhsj))) |
2848
da7e6655cd4c
fixed the problem when giving a complex default-term; the fundef lemmas in Nominal_Base were not general enough
Christian Urban <urbanc@in.tum.de>
parents:
2822
diff
changeset
|
297 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
298 |
in if j < i then |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
299 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
300 |
val compat = lookup_compat_thm j i cts |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
301 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
302 |
compat (* "!!qj qi. Gsj => Gsi => lhsj = lhsi ==> rhsj = rhsi" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
303 |
|> fold Thm.forall_elim (cqsj @ cqsi) (* "Gsj => Gsi => lhsj = lhsi ==> rhsj = rhsi" *) |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
304 |
|> fold Thm.elim_implies eqvtsj (* nominal *) |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
305 |
|> fold Thm.elim_implies eqvtsi (* nominal *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
306 |
|> fold Thm.elim_implies invsj (* nominal *) |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
307 |
|> fold Thm.elim_implies invsi (* nominal *) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
308 |
|> fold Thm.elim_implies agsj |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
309 |
|> fold Thm.elim_implies agsi |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
310 |
|> Thm.elim_implies ((Thm.assume lhsi_eq_lhsj) RS sym) (* "Gsj, Gsi, lhsi = lhsj |-- rhsj = rhsi" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
311 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
312 |
else |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
313 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
314 |
val compat = lookup_compat_thm i j cts |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
315 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
316 |
compat (* "!!qi qj. Gsi => Gsj => lhsi = lhsj ==> rhsi = rhsj" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
317 |
|> fold Thm.forall_elim (cqsi @ cqsj) (* "Gsi => Gsj => lhsi = lhsj ==> rhsi = rhsj" *) |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
318 |
|> fold Thm.elim_implies eqvtsi (* nominal *) |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
319 |
|> fold Thm.elim_implies eqvtsj (* nominal *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
320 |
|> fold Thm.elim_implies invsi (* nominal *) |
2862
47063163f333
added eqvt_at and invariant for boths sides of the equations
Christian Urban <urbanc@in.tum.de>
parents:
2848
diff
changeset
|
321 |
|> fold Thm.elim_implies invsj (* nominal *) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
322 |
|> fold Thm.elim_implies agsi |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
323 |
|> fold Thm.elim_implies agsj |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
324 |
|> Thm.elim_implies (Thm.assume lhsi_eq_lhsj) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
325 |
|> (fn thm => thm RS sym) (* "Gsi, Gsj, lhsi = lhsj |-- rhsj = rhsi" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
326 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
327 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
328 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
329 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
330 |
(* Generates the replacement lemma in fully quantified form. *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
331 |
fun mk_replacement_lemma thy h ih_elim clause = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
332 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
333 |
val ClauseInfo {cdata=ClauseContext {qs, lhs, cqs, ags, case_hyp, ...}, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
334 |
RCs, tree, ...} = clause |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
335 |
local open Conv in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
336 |
val ih_conv = arg1_conv o arg_conv o arg_conv |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
337 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
338 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
339 |
val ih_elim_case = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
340 |
Conv.fconv_rule (ih_conv (K (case_hyp RS eq_reflection))) ih_elim |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
341 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
342 |
val Ris = map (fn RCInfo {llRI, ...} => llRI) RCs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
343 |
val h_assums = map (fn RCInfo {h_assum, ...} => |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
344 |
Thm.assume (cterm_of thy (subst_bounds (rev qs, h_assum)))) RCs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
345 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
346 |
val (eql, _) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
347 |
Function_Ctx_Tree.rewrite_by_tree thy h ih_elim_case (Ris ~~ h_assums) tree |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
348 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
349 |
val replace_lemma = (eql RS meta_eq_to_obj_eq) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
350 |
|> Thm.implies_intr (cprop_of case_hyp) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
351 |
|> fold_rev (Thm.implies_intr o cprop_of) h_assums |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
352 |
|> fold_rev (Thm.implies_intr o cprop_of) ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
353 |
|> fold_rev Thm.forall_intr cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
354 |
|> Thm.close_derivation |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
355 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
356 |
replace_lemma |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
357 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
358 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
359 |
(* nominal *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
360 |
(* Generates the eqvt lemmas for each clause *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
361 |
fun mk_eqvt_lemma thy ih_eqvt clause = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
362 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
363 |
val ClauseInfo {cdata=ClauseContext {cqs, ags, case_hyp, ...}, RCs, ...} = clause |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
364 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
365 |
local open Conv in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
366 |
val ih_conv = arg1_conv o arg_conv o arg_conv |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
367 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
368 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
369 |
val ih_eqvt_case = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
370 |
Conv.fconv_rule (ih_conv (K (case_hyp RS eq_reflection))) ih_eqvt |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
371 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
372 |
fun prep_eqvt (RCInfo {llRI, RIvs, CCas, ...}) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
373 |
(llRI RS ih_eqvt_case) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
374 |
|> fold_rev (Thm.implies_intr o cprop_of) CCas |
2802
3b9ef98a03d2
first test to fix the problem with free variables
Christian Urban <urbanc@in.tum.de>
parents:
2796
diff
changeset
|
375 |
|> fold_rev (Thm.forall_intr o cterm_of thy o Free) RIvs |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
376 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
377 |
map prep_eqvt RCs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
378 |
|> map (fold_rev (Thm.implies_intr o cprop_of) ags) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
379 |
|> map (Thm.implies_intr (cprop_of case_hyp)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
380 |
|> map (fold_rev Thm.forall_intr cqs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
381 |
|> map (Thm.close_derivation) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
382 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
383 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
384 |
(* nominal *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
385 |
fun mk_invariant_lemma thy ih_inv clause = |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
386 |
let |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
387 |
val ClauseInfo {cdata=ClauseContext {cqs, ags, case_hyp, ...}, RCs, ...} = clause |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
388 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
389 |
local open Conv in |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
390 |
val ih_conv = arg1_conv o arg_conv o arg_conv |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
391 |
end |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
392 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
393 |
val ih_inv_case = |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
394 |
Conv.fconv_rule (ih_conv (K (case_hyp RS eq_reflection))) ih_inv |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
395 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
396 |
fun prep_inv (RCInfo {llRI, RIvs, CCas, ...}) = |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
397 |
(llRI RS ih_inv_case) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
398 |
|> fold_rev (Thm.implies_intr o cprop_of) CCas |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
399 |
|> fold_rev (Thm.forall_intr o cterm_of thy o Free) RIvs |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
400 |
in |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
401 |
map prep_inv RCs |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
402 |
|> map (fold_rev (Thm.implies_intr o cprop_of) ags) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
403 |
|> map (Thm.implies_intr (cprop_of case_hyp)) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
404 |
|> map (fold_rev Thm.forall_intr cqs) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
405 |
|> map (Thm.close_derivation) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
406 |
end |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
407 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
408 |
(* nominal *) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
409 |
fun mk_uniqueness_clause thy globals compat_store eqvts invs clausei clausej RLj = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
410 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
411 |
val Globals {h, y, x, fvar, ...} = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
412 |
val ClauseInfo {no=i, cdata=cctxi as ClauseContext {ctxt=ctxti, lhs=lhsi, case_hyp, cqs = cqsi, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
413 |
ags = agsi, ...}, ...} = clausei |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
414 |
val ClauseInfo {no=j, qglr=cdescj, RCs=RCsj, ...} = clausej |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
415 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
416 |
val cctxj as ClauseContext {ags = agsj', lhs = lhsj', rhs = rhsj', qs = qsj', cqs = cqsj', ...} = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
417 |
mk_clause_context x ctxti cdescj |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
418 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
419 |
val rhsj'h = Pattern.rewrite_term thy [(fvar,h)] [] rhsj' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
420 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
421 |
val Ghsj' = map |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
422 |
(fn RCInfo {h_assum, ...} => Thm.assume (cterm_of thy (subst_bounds (rev qsj', h_assum)))) RCsj |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
423 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
424 |
val y_eq_rhsj'h = Thm.assume (cterm_of thy (HOLogic.mk_Trueprop (mk_eq (y, rhsj'h)))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
425 |
val lhsi_eq_lhsj' = Thm.assume (cterm_of thy (HOLogic.mk_Trueprop (mk_eq (lhsi, lhsj')))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
426 |
(* lhs_i = lhs_j' |-- lhs_i = lhs_j' *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
427 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
428 |
val case_hypj' = trans OF [case_hyp, lhsi_eq_lhsj'] |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
429 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
430 |
val RLj_import = RLj |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
431 |
|> fold Thm.forall_elim cqsj' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
432 |
|> fold Thm.elim_implies agsj' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
433 |
|> fold Thm.elim_implies Ghsj' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
434 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
435 |
val eqvtsi = nth eqvts (i - 1) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
436 |
|> map (fold Thm.forall_elim cqsi) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
437 |
|> map (fold Thm.elim_implies [case_hyp]) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
438 |
|> map (fold Thm.elim_implies agsi) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
439 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
440 |
val eqvtsj = nth eqvts (j - 1) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
441 |
|> map (fold Thm.forall_elim cqsj') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
442 |
|> map (fold Thm.elim_implies [case_hypj']) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
443 |
|> map (fold Thm.elim_implies agsj') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
444 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
445 |
val invsi = nth invs (i - 1) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
446 |
|> map (fold Thm.forall_elim cqsi) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
447 |
|> map (fold Thm.elim_implies [case_hyp]) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
448 |
|> map (fold Thm.elim_implies agsi) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
449 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
450 |
val invsj = nth invs (j - 1) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
451 |
|> map (fold Thm.forall_elim cqsj') |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
452 |
|> map (fold Thm.elim_implies [case_hypj']) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
453 |
|> map (fold Thm.elim_implies agsj') |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
454 |
|
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
455 |
val compat = get_compat_thm thy compat_store eqvtsi eqvtsj invsi invsj i j cctxi cctxj |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
456 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
457 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
458 |
(trans OF [case_hyp, lhsi_eq_lhsj']) (* lhs_i = lhs_j' |-- x = lhs_j' *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
459 |
|> Thm.implies_elim RLj_import |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
460 |
(* Rj1' ... Rjk', lhs_i = lhs_j' |-- rhs_j'_h = rhs_j'_f *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
461 |
|> (fn it => trans OF [it, compat]) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
462 |
(* lhs_i = lhs_j', Gj', Rj1' ... Rjk' |-- rhs_j'_h = rhs_i_f *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
463 |
|> (fn it => trans OF [y_eq_rhsj'h, it]) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
464 |
(* lhs_i = lhs_j', Gj', Rj1' ... Rjk', y = rhs_j_h' |-- y = rhs_i_f *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
465 |
|> fold_rev (Thm.implies_intr o cprop_of) Ghsj' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
466 |
|> fold_rev (Thm.implies_intr o cprop_of) agsj' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
467 |
(* lhs_i = lhs_j' , y = rhs_j_h' |-- Gj', Rj1'...Rjk' ==> y = rhs_i_f *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
468 |
|> Thm.implies_intr (cprop_of y_eq_rhsj'h) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
469 |
|> Thm.implies_intr (cprop_of lhsi_eq_lhsj') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
470 |
|> fold_rev Thm.forall_intr (cterm_of thy h :: cqsj') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
471 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
472 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
473 |
(* nominal *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
474 |
fun mk_uniqueness_case thy globals G f ihyp ih_intro G_cases compat_store clauses replems eqvtlems invlems |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
475 |
clausei = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
476 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
477 |
val Globals {x, y, ranT, fvar, ...} = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
478 |
val ClauseInfo {cdata = ClauseContext {lhs, rhs, cqs, ags, case_hyp, ...}, lGI, RCs, ...} = clausei |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
479 |
val rhsC = Pattern.rewrite_term thy [(fvar, f)] [] rhs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
480 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
481 |
val ih_intro_case = full_simplify (HOL_basic_ss addsimps [case_hyp]) ih_intro |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
482 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
483 |
fun prep_RC (RCInfo {llRI, RIvs, CCas, ...}) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
484 |
(llRI RS ih_intro_case) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
485 |
|> fold_rev (Thm.implies_intr o cprop_of) CCas |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
486 |
|> fold_rev (Thm.forall_intr o cterm_of thy o Free) RIvs |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
487 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
488 |
val existence = fold (curry op COMP o prep_RC) RCs lGI |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
489 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
490 |
val P = cterm_of thy (mk_eq (y, rhsC)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
491 |
val G_lhs_y = Thm.assume (cterm_of thy (HOLogic.mk_Trueprop (G $ lhs $ y))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
492 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
493 |
val unique_clauses = |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
494 |
map2 (mk_uniqueness_clause thy globals compat_store eqvtlems invlems clausei) clauses replems |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
495 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
496 |
fun elim_implies_eta A AB = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
497 |
Thm.compose_no_flatten true (A, 0) 1 AB |> Seq.list_of |> the_single |
2789
32979078bfe9
functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Christian Urban <urbanc@in.tum.de>
parents:
2788
diff
changeset
|
498 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
499 |
val uniqueness = G_cases |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
500 |
|> Thm.forall_elim (cterm_of thy lhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
501 |
|> Thm.forall_elim (cterm_of thy y) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
502 |
|> Thm.forall_elim P |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
503 |
|> Thm.elim_implies G_lhs_y |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
504 |
|> fold elim_implies_eta unique_clauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
505 |
|> Thm.implies_intr (cprop_of G_lhs_y) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
506 |
|> Thm.forall_intr (cterm_of thy y) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
507 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
508 |
val P2 = cterm_of thy (lambda y (G $ lhs $ y)) (* P2 y := (lhs, y): G *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
509 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
510 |
val exactly_one = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
511 |
ex1I |> instantiate' [SOME (ctyp_of thy ranT)] [SOME P2, SOME (cterm_of thy rhsC)] |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
512 |
|> curry (op COMP) existence |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
513 |
|> curry (op COMP) uniqueness |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
514 |
|> simplify (HOL_basic_ss addsimps [case_hyp RS sym]) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
515 |
|> Thm.implies_intr (cprop_of case_hyp) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
516 |
|> fold_rev (Thm.implies_intr o cprop_of) ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
517 |
|> fold_rev Thm.forall_intr cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
518 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
519 |
val function_value = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
520 |
existence |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
521 |
|> Thm.implies_intr ihyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
522 |
|> Thm.implies_intr (cprop_of case_hyp) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
523 |
|> Thm.forall_intr (cterm_of thy x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
524 |
|> Thm.forall_elim (cterm_of thy lhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
525 |
|> curry (op RS) refl |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
526 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
527 |
(exactly_one, function_value) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
528 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
529 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
530 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
531 |
(* nominal *) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
532 |
fun prove_stuff ctxt globals G f R clauses complete compat compat_store G_elim G_eqvt invariant f_def = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
533 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
534 |
val Globals {h, domT, ranT, x, ...} = globals |
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
535 |
val thy = Proof_Context.theory_of ctxt |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
536 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
537 |
(* Inductive Hypothesis: !!z. (z,x):R ==> EX!y. (z,y):G *) |
3108
61db5ad429bb
updated to Isabelle 16 January
Christian Urban <urbanc@in.tum.de>
parents:
3045
diff
changeset
|
538 |
val ihyp = Logic.all_const domT $ Abs ("z", domT, |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
539 |
Logic.mk_implies (HOLogic.mk_Trueprop (R $ Bound 0 $ x), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
540 |
HOLogic.mk_Trueprop (Const (@{const_name Ex1}, (ranT --> boolT) --> boolT) $ |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
541 |
Abs ("y", ranT, G $ Bound 1 $ Bound 0)))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
542 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
543 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
544 |
val ihyp_thm = Thm.assume ihyp |> Thm.forall_elim_vars 0 |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
545 |
val ih_intro = ihyp_thm RS (f_def RS ex1_implies_ex) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
546 |
val ih_elim = ihyp_thm RS (f_def RS ex1_implies_un) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
547 |
|> instantiate' [] [NONE, SOME (cterm_of thy h)] |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
548 |
val ih_eqvt = ihyp_thm RS (G_eqvt RS (f_def RS @{thm fundef_ex1_eqvt_at})) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
549 |
val ih_inv = ihyp_thm RS (invariant COMP (f_def RS @{thm fundef_ex1_prop})) |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
550 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
551 |
val _ = trace_msg (K "Proving Replacement lemmas...") |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
552 |
val repLemmas = map (mk_replacement_lemma thy h ih_elim) clauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
553 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
554 |
val _ = trace_msg (K "Proving Equivariance lemmas...") |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
555 |
val eqvtLemmas = map (mk_eqvt_lemma thy ih_eqvt) clauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
556 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
557 |
val _ = trace_msg (K "Proving Invariance lemmas...") |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
558 |
val invLemmas = map (mk_invariant_lemma thy ih_inv) clauses |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
559 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
560 |
val _ = trace_msg (K "Proving cases for unique existence...") |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
561 |
val (ex1s, values) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
562 |
split_list (map (mk_uniqueness_case thy globals G f |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
563 |
ihyp ih_intro G_elim compat_store clauses repLemmas eqvtLemmas invLemmas) clauses) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
564 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
565 |
val _ = trace_msg (K "Proving: Graph is a function") |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
566 |
val graph_is_function = complete |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
567 |
|> Thm.forall_elim_vars 0 |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
568 |
|> fold (curry op COMP) ex1s |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
569 |
|> Thm.implies_intr (ihyp) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
570 |
|> Thm.implies_intr (cterm_of thy (HOLogic.mk_Trueprop (mk_acc domT R $ x))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
571 |
|> Thm.forall_intr (cterm_of thy x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
572 |
|> (fn it => Drule.compose_single (it, 2, acc_induct_rule)) (* "EX! y. (?x,y):G" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
573 |
|> (fn it => fold (Thm.forall_intr o cterm_of thy o Var) (Term.add_vars (prop_of it) []) it) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
574 |
|
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
575 |
val goalstate = |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
576 |
Conjunction.intr (Conjunction.intr (Conjunction.intr graph_is_function complete) invariant) G_eqvt |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
577 |
|> Thm.close_derivation |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
578 |
|> Goal.protect |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
579 |
|> fold_rev (Thm.implies_intr o cprop_of) compat |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
580 |
|> Thm.implies_intr (cprop_of complete) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
581 |
|> Thm.implies_intr (cprop_of invariant) |
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
582 |
|> Thm.implies_intr (cprop_of G_eqvt) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
583 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
584 |
(goalstate, values) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
585 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
586 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
587 |
(* wrapper -- restores quantifiers in rule specifications *) |
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
588 |
fun inductive_def (binding as ((R, T), _)) intrs lthy = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
589 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
590 |
val ({intrs = intrs_gen, elims = [elim_gen], preds = [ Rdef ], induct, raw_induct, ...}, lthy) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
591 |
lthy |
2885
1264f2a21ea9
some rudimentary infrastructure for storing data about nominal datatypes
Christian Urban <urbanc@in.tum.de>
parents:
2862
diff
changeset
|
592 |
|> Local_Theory.conceal |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
593 |
|> Inductive.add_inductive_i |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
594 |
{quiet_mode = true, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
595 |
verbose = ! trace, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
596 |
alt_name = Binding.empty, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
597 |
coind = false, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
598 |
no_elim = false, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
599 |
no_ind = false, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
600 |
skip_mono = true, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
601 |
fork_mono = false} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
602 |
[binding] (* relation *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
603 |
[] (* no parameters *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
604 |
(map (fn t => (Attrib.empty_binding, t)) intrs) (* intro rules *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
605 |
[] (* no special monos *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
606 |
||> Local_Theory.restore_naming lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
607 |
|
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
608 |
val cert = cterm_of (Proof_Context.theory_of lthy) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
609 |
fun requantify orig_intro thm = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
610 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
611 |
val (qs, t) = dest_all_all orig_intro |
2781
542ff50555f5
updated to new Isabelle (> 9 May)
Christian Urban <urbanc@in.tum.de>
parents:
2745
diff
changeset
|
612 |
val frees = Variable.add_frees lthy t [] |> remove (op =) (Binding.name_of R, T) |
542ff50555f5
updated to new Isabelle (> 9 May)
Christian Urban <urbanc@in.tum.de>
parents:
2745
diff
changeset
|
613 |
val vars = Term.add_vars (prop_of thm) [] |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
614 |
val varmap = AList.lookup (op =) (frees ~~ map fst vars) |
2781
542ff50555f5
updated to new Isabelle (> 9 May)
Christian Urban <urbanc@in.tum.de>
parents:
2745
diff
changeset
|
615 |
#> the_default ("",0) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
616 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
617 |
fold_rev (fn Free (n, T) => |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
618 |
forall_intr_rename (n, cert (Var (varmap (n, T), T)))) qs thm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
619 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
620 |
in |
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
621 |
((Rdef, map2 requantify intrs intrs_gen, forall_intr_vars elim_gen, induct), lthy) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
622 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
623 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
624 |
(* nominal *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
625 |
fun define_graph Gname fvar domT ranT clauses RCss lthy = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
626 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
627 |
val GT = domT --> ranT --> boolT |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
628 |
val (Gvar as (n, T)) = singleton (Variable.variant_frees lthy []) (Gname, GT) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
629 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
630 |
fun mk_GIntro (ClauseContext {qs, gs, lhs, rhs, ...}) RCs = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
631 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
632 |
fun mk_h_assm (rcfix, rcassm, rcarg) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
633 |
HOLogic.mk_Trueprop (Free Gvar $ rcarg $ (fvar $ rcarg)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
634 |
|> fold_rev (curry Logic.mk_implies o prop_of) rcassm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
635 |
|> fold_rev (Logic.all o Free) rcfix |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
636 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
637 |
HOLogic.mk_Trueprop (Free Gvar $ lhs $ rhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
638 |
|> fold_rev (curry Logic.mk_implies o mk_h_assm) RCs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
639 |
|> fold_rev (curry Logic.mk_implies) gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
640 |
|> fold_rev Logic.all (fvar :: qs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
641 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
642 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
643 |
val G_intros = map2 mk_GIntro clauses RCss |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
644 |
in |
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
645 |
inductive_def ((Binding.name n, T), NoSyn) G_intros lthy |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
646 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
647 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
648 |
fun define_function fdefname (fname, mixfix) domT ranT G default lthy = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
649 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
650 |
val f_def = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
651 |
Abs ("x", domT, Const (@{const_name FunDef.THE_default}, ranT --> (ranT --> boolT) --> ranT) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
652 |
$ (default $ Bound 0) $ Abs ("y", ranT, G $ Bound 1 $ Bound 0)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
653 |
|> Syntax.check_term lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
654 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
655 |
Local_Theory.define |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
656 |
((Binding.name (function_name fname), mixfix), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
657 |
((Binding.conceal (Binding.name fdefname), []), f_def)) lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
658 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
659 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
660 |
(* nominal *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
661 |
fun define_recursion_relation Rname domT qglrs clauses RCss lthy = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
662 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
663 |
val RT = domT --> domT --> boolT |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
664 |
val (Rvar as (n, T)) = singleton (Variable.variant_frees lthy []) (Rname, RT) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
665 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
666 |
fun mk_RIntro (ClauseContext {qs, gs, lhs, ...}, (oqs, _, _, _)) (rcfix, rcassm, rcarg) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
667 |
HOLogic.mk_Trueprop (Free Rvar $ rcarg $ lhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
668 |
|> fold_rev (curry Logic.mk_implies o prop_of) rcassm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
669 |
|> fold_rev (curry Logic.mk_implies) gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
670 |
|> fold_rev (Logic.all o Free) rcfix |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
671 |
|> fold_rev mk_forall_rename (map fst oqs ~~ qs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
672 |
(* "!!qs xs. CS ==> G => (r, lhs) : R" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
673 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
674 |
val R_intross = map2 (map o mk_RIntro) (clauses ~~ qglrs) RCss |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
675 |
|
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
676 |
val ((R, RIntro_thms, R_elim, _), lthy) = |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
677 |
inductive_def ((Binding.name n, T), NoSyn) (flat R_intross) lthy |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
678 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
679 |
((R, Library.unflat R_intross RIntro_thms, R_elim), lthy) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
680 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
681 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
682 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
683 |
fun fix_globals domT ranT fvar ctxt = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
684 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
685 |
val ([h, y, x, z, a, D, P, Pbool],ctxt') = Variable.variant_fixes |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
686 |
["h_fd", "y_fd", "x_fd", "z_fd", "a_fd", "D_fd", "P_fd", "Pb_fd"] ctxt |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
687 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
688 |
(Globals {h = Free (h, domT --> ranT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
689 |
y = Free (y, ranT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
690 |
x = Free (x, domT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
691 |
z = Free (z, domT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
692 |
a = Free (a, domT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
693 |
D = Free (D, domT --> boolT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
694 |
P = Free (P, domT --> boolT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
695 |
Pbool = Free (Pbool, boolT), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
696 |
fvar = fvar, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
697 |
domT = domT, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
698 |
ranT = ranT}, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
699 |
ctxt') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
700 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
701 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
702 |
fun inst_RC thy fvar f (rcfix, rcassm, rcarg) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
703 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
704 |
fun inst_term t = subst_bound(f, abstract_over (fvar, t)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
705 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
706 |
(rcfix, map (Thm.assume o cterm_of thy o inst_term o prop_of) rcassm, inst_term rcarg) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
707 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
708 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
709 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
710 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
711 |
(********************************************************** |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
712 |
* PROVING THE RULES |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
713 |
**********************************************************) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
714 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
715 |
fun mk_psimps thy globals R clauses valthms f_iff graph_is_function = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
716 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
717 |
val Globals {domT, z, ...} = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
718 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
719 |
fun mk_psimp (ClauseInfo {qglr = (oqs, _, _, _), cdata = ClauseContext {cqs, lhs, ags, ...}, ...}) valthm = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
720 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
721 |
val lhs_acc = cterm_of thy (HOLogic.mk_Trueprop (mk_acc domT R $ lhs)) (* "acc R lhs" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
722 |
val z_smaller = cterm_of thy (HOLogic.mk_Trueprop (R $ z $ lhs)) (* "R z lhs" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
723 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
724 |
((Thm.assume z_smaller) RS ((Thm.assume lhs_acc) RS acc_downward)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
725 |
|> (fn it => it COMP graph_is_function) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
726 |
|> Thm.implies_intr z_smaller |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
727 |
|> Thm.forall_intr (cterm_of thy z) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
728 |
|> (fn it => it COMP valthm) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
729 |
|> Thm.implies_intr lhs_acc |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
730 |
|> asm_simplify (HOL_basic_ss addsimps [f_iff]) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
731 |
|> fold_rev (Thm.implies_intr o cprop_of) ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
732 |
|> fold_rev forall_intr_rename (map fst oqs ~~ cqs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
733 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
734 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
735 |
map2 mk_psimp clauses valthms |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
736 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
737 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
738 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
739 |
(** Induction rule **) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
740 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
741 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
742 |
val acc_subset_induct = @{thm predicate1I} RS @{thm accp_subset_induct} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
743 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
744 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
745 |
fun mk_partial_induct_rule thy globals R complete_thm clauses = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
746 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
747 |
val Globals {domT, x, z, a, P, D, ...} = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
748 |
val acc_R = mk_acc domT R |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
749 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
750 |
val x_D = Thm.assume (cterm_of thy (HOLogic.mk_Trueprop (D $ x))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
751 |
val a_D = cterm_of thy (HOLogic.mk_Trueprop (D $ a)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
752 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
753 |
val D_subset = cterm_of thy (Logic.all x |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
754 |
(Logic.mk_implies (HOLogic.mk_Trueprop (D $ x), HOLogic.mk_Trueprop (acc_R $ x)))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
755 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
756 |
val D_dcl = (* "!!x z. [| x: D; (z,x):R |] ==> z:D" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
757 |
Logic.all x (Logic.all z (Logic.mk_implies (HOLogic.mk_Trueprop (D $ x), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
758 |
Logic.mk_implies (HOLogic.mk_Trueprop (R $ z $ x), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
759 |
HOLogic.mk_Trueprop (D $ z))))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
760 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
761 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
762 |
(* Inductive Hypothesis: !!z. (z,x):R ==> P z *) |
3108
61db5ad429bb
updated to Isabelle 16 January
Christian Urban <urbanc@in.tum.de>
parents:
3045
diff
changeset
|
763 |
val ihyp = Logic.all_const domT $ Abs ("z", domT, |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
764 |
Logic.mk_implies (HOLogic.mk_Trueprop (R $ Bound 0 $ x), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
765 |
HOLogic.mk_Trueprop (P $ Bound 0))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
766 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
767 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
768 |
val aihyp = Thm.assume ihyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
769 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
770 |
fun prove_case clause = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
771 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
772 |
val ClauseInfo {cdata = ClauseContext {ctxt, qs, cqs, ags, gs, lhs, case_hyp, ...}, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
773 |
RCs, qglr = (oqs, _, _, _), ...} = clause |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
774 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
775 |
val case_hyp_conv = K (case_hyp RS eq_reflection) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
776 |
local open Conv in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
777 |
val lhs_D = fconv_rule (arg_conv (arg_conv (case_hyp_conv))) x_D |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
778 |
val sih = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
779 |
fconv_rule (Conv.binder_conv |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
780 |
(K (arg1_conv (arg_conv (arg_conv case_hyp_conv)))) ctxt) aihyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
781 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
782 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
783 |
fun mk_Prec (RCInfo {llRI, RIvs, CCas, rcarg, ...}) = sih |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
784 |
|> Thm.forall_elim (cterm_of thy rcarg) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
785 |
|> Thm.elim_implies llRI |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
786 |
|> fold_rev (Thm.implies_intr o cprop_of) CCas |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
787 |
|> fold_rev (Thm.forall_intr o cterm_of thy o Free) RIvs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
788 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
789 |
val P_recs = map mk_Prec RCs (* [P rec1, P rec2, ... ] *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
790 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
791 |
val step = HOLogic.mk_Trueprop (P $ lhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
792 |
|> fold_rev (curry Logic.mk_implies o prop_of) P_recs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
793 |
|> fold_rev (curry Logic.mk_implies) gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
794 |
|> curry Logic.mk_implies (HOLogic.mk_Trueprop (D $ lhs)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
795 |
|> fold_rev mk_forall_rename (map fst oqs ~~ qs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
796 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
797 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
798 |
val P_lhs = Thm.assume step |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
799 |
|> fold Thm.forall_elim cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
800 |
|> Thm.elim_implies lhs_D |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
801 |
|> fold Thm.elim_implies ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
802 |
|> fold Thm.elim_implies P_recs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
803 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
804 |
val res = cterm_of thy (HOLogic.mk_Trueprop (P $ x)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
805 |
|> Conv.arg_conv (Conv.arg_conv case_hyp_conv) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
806 |
|> Thm.symmetric (* P lhs == P x *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
807 |
|> (fn eql => Thm.equal_elim eql P_lhs) (* "P x" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
808 |
|> Thm.implies_intr (cprop_of case_hyp) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
809 |
|> fold_rev (Thm.implies_intr o cprop_of) ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
810 |
|> fold_rev Thm.forall_intr cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
811 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
812 |
(res, step) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
813 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
814 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
815 |
val (cases, steps) = split_list (map prove_case clauses) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
816 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
817 |
val istep = complete_thm |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
818 |
|> Thm.forall_elim_vars 0 |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
819 |
|> fold (curry op COMP) cases (* P x *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
820 |
|> Thm.implies_intr ihyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
821 |
|> Thm.implies_intr (cprop_of x_D) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
822 |
|> Thm.forall_intr (cterm_of thy x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
823 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
824 |
val subset_induct_rule = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
825 |
acc_subset_induct |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
826 |
|> (curry op COMP) (Thm.assume D_subset) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
827 |
|> (curry op COMP) (Thm.assume D_dcl) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
828 |
|> (curry op COMP) (Thm.assume a_D) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
829 |
|> (curry op COMP) istep |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
830 |
|> fold_rev Thm.implies_intr steps |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
831 |
|> Thm.implies_intr a_D |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
832 |
|> Thm.implies_intr D_dcl |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
833 |
|> Thm.implies_intr D_subset |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
834 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
835 |
val simple_induct_rule = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
836 |
subset_induct_rule |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
837 |
|> Thm.forall_intr (cterm_of thy D) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
838 |
|> Thm.forall_elim (cterm_of thy acc_R) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
839 |
|> assume_tac 1 |> Seq.hd |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
840 |
|> (curry op COMP) (acc_downward |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
841 |
|> (instantiate' [SOME (ctyp_of thy domT)] |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
842 |
(map (SOME o cterm_of thy) [R, x, z])) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
843 |
|> Thm.forall_intr (cterm_of thy z) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
844 |
|> Thm.forall_intr (cterm_of thy x)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
845 |
|> Thm.forall_intr (cterm_of thy a) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
846 |
|> Thm.forall_intr (cterm_of thy P) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
847 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
848 |
simple_induct_rule |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
849 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
850 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
851 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
852 |
(* FIXME: broken by design *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
853 |
fun mk_domain_intro ctxt (Globals {domT, ...}) R R_cases clause = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
854 |
let |
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
855 |
val thy = Proof_Context.theory_of ctxt |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
856 |
val ClauseInfo {cdata = ClauseContext {gs, lhs, cqs, ...}, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
857 |
qglr = (oqs, _, _, _), ...} = clause |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
858 |
val goal = HOLogic.mk_Trueprop (mk_acc domT R $ lhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
859 |
|> fold_rev (curry Logic.mk_implies) gs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
860 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
861 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
862 |
Goal.init goal |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
863 |
|> (SINGLE (resolve_tac [accI] 1)) |> the |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
864 |
|> (SINGLE (eresolve_tac [Thm.forall_elim_vars 0 R_cases] 1)) |> the |
2788
036a19936feb
updated to new Isabelle
Christian Urban <urbanc@in.tum.de>
parents:
2781
diff
changeset
|
865 |
|> (SINGLE (auto_tac ctxt)) |> the |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
866 |
|> Goal.conclude |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
867 |
|> fold_rev forall_intr_rename (map fst oqs ~~ cqs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
868 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
869 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
870 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
871 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
872 |
(** Termination rule **) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
873 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
874 |
val wf_induct_rule = @{thm Wellfounded.wfP_induct_rule} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
875 |
val wf_in_rel = @{thm FunDef.wf_in_rel} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
876 |
val in_rel_def = @{thm FunDef.in_rel_def} |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
877 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
878 |
fun mk_nest_term_case thy globals R' ihyp clause = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
879 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
880 |
val Globals {z, ...} = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
881 |
val ClauseInfo {cdata = ClauseContext {qs, cqs, ags, lhs, case_hyp, ...}, tree, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
882 |
qglr=(oqs, _, _, _), ...} = clause |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
883 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
884 |
val ih_case = full_simplify (HOL_basic_ss addsimps [case_hyp]) ihyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
885 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
886 |
fun step (fixes, assumes) (_ $ arg) u (sub,(hyps,thms)) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
887 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
888 |
val used = (u @ sub) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
889 |
|> map (fn (ctx,thm) => Function_Ctx_Tree.export_thm thy ctx thm) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
890 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
891 |
val hyp = HOLogic.mk_Trueprop (R' $ arg $ lhs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
892 |
|> fold_rev (curry Logic.mk_implies o prop_of) used (* additional hyps *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
893 |
|> Function_Ctx_Tree.export_term (fixes, assumes) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
894 |
|> fold_rev (curry Logic.mk_implies o prop_of) ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
895 |
|> fold_rev mk_forall_rename (map fst oqs ~~ qs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
896 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
897 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
898 |
val thm = Thm.assume hyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
899 |
|> fold Thm.forall_elim cqs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
900 |
|> fold Thm.elim_implies ags |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
901 |
|> Function_Ctx_Tree.import_thm thy (fixes, assumes) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
902 |
|> fold Thm.elim_implies used (* "(arg, lhs) : R'" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
903 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
904 |
val z_eq_arg = HOLogic.mk_Trueprop (mk_eq (z, arg)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
905 |
|> cterm_of thy |> Thm.assume |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
906 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
907 |
val acc = thm COMP ih_case |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
908 |
val z_acc_local = acc |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
909 |
|> Conv.fconv_rule |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
910 |
(Conv.arg_conv (Conv.arg_conv (K (Thm.symmetric (z_eq_arg RS eq_reflection))))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
911 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
912 |
val ethm = z_acc_local |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
913 |
|> Function_Ctx_Tree.export_thm thy (fixes, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
914 |
z_eq_arg :: case_hyp :: ags @ assumes) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
915 |
|> fold_rev forall_intr_rename (map fst oqs ~~ cqs) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
916 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
917 |
val sub' = sub @ [(([],[]), acc)] |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
918 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
919 |
(sub', (hyp :: hyps, ethm :: thms)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
920 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
921 |
| step _ _ _ _ = raise Match |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
922 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
923 |
Function_Ctx_Tree.traverse_tree step tree |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
924 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
925 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
926 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
927 |
fun mk_nest_term_rule thy globals R R_cases clauses = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
928 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
929 |
val Globals { domT, x, z, ... } = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
930 |
val acc_R = mk_acc domT R |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
931 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
932 |
val R' = Free ("R", fastype_of R) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
933 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
934 |
val Rrel = Free ("R", HOLogic.mk_setT (HOLogic.mk_prodT (domT, domT))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
935 |
val inrel_R = Const (@{const_name FunDef.in_rel}, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
936 |
HOLogic.mk_setT (HOLogic.mk_prodT (domT, domT)) --> fastype_of R) $ Rrel |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
937 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
938 |
val wfR' = HOLogic.mk_Trueprop (Const (@{const_name Wellfounded.wfP}, |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
939 |
(domT --> domT --> boolT) --> boolT) $ R') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
940 |
|> cterm_of thy (* "wf R'" *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
941 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
942 |
(* Inductive Hypothesis: !!z. (z,x):R' ==> z : acc R *) |
3108
61db5ad429bb
updated to Isabelle 16 January
Christian Urban <urbanc@in.tum.de>
parents:
3045
diff
changeset
|
943 |
val ihyp = Logic.all_const domT $ Abs ("z", domT, |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
944 |
Logic.mk_implies (HOLogic.mk_Trueprop (R' $ Bound 0 $ x), |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
945 |
HOLogic.mk_Trueprop (acc_R $ Bound 0))) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
946 |
|> cterm_of thy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
947 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
948 |
val ihyp_a = Thm.assume ihyp |> Thm.forall_elim_vars 0 |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
949 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
950 |
val R_z_x = cterm_of thy (HOLogic.mk_Trueprop (R $ z $ x)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
951 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
952 |
val (hyps, cases) = fold (mk_nest_term_case thy globals R' ihyp_a) clauses ([], []) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
953 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
954 |
R_cases |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
955 |
|> Thm.forall_elim (cterm_of thy z) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
956 |
|> Thm.forall_elim (cterm_of thy x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
957 |
|> Thm.forall_elim (cterm_of thy (acc_R $ z)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
958 |
|> curry op COMP (Thm.assume R_z_x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
959 |
|> fold_rev (curry op COMP) cases |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
960 |
|> Thm.implies_intr R_z_x |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
961 |
|> Thm.forall_intr (cterm_of thy z) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
962 |
|> (fn it => it COMP accI) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
963 |
|> Thm.implies_intr ihyp |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
964 |
|> Thm.forall_intr (cterm_of thy x) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
965 |
|> (fn it => Drule.compose_single(it,2,wf_induct_rule)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
966 |
|> curry op RS (Thm.assume wfR') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
967 |
|> forall_intr_vars |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
968 |
|> (fn it => it COMP allI) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
969 |
|> fold Thm.implies_intr hyps |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
970 |
|> Thm.implies_intr wfR' |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
971 |
|> Thm.forall_intr (cterm_of thy R') |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
972 |
|> Thm.forall_elim (cterm_of thy (inrel_R)) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
973 |
|> curry op RS wf_in_rel |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
974 |
|> full_simplify (HOL_basic_ss addsimps [in_rel_def]) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
975 |
|> Thm.forall_intr (cterm_of thy Rrel) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
976 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
977 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
978 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
979 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
980 |
(* nominal *) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
981 |
fun prepare_nominal_function config defname [((fname, fT), mixfix)] abstract_qglrs lthy = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
982 |
let |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
983 |
val NominalFunctionConfig {domintros, default=default_opt, inv=invariant_opt,...} = config |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
984 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
985 |
val default_str = the_default "%x. undefined" default_opt (*FIXME dynamic scoping*) |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
986 |
val invariant_str = the_default "%x y. True" invariant_opt |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
987 |
val fvar = Free (fname, fT) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
988 |
val domT = domain_type fT |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
989 |
val ranT = range_type fT |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
990 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
991 |
val default = Syntax.parse_term lthy default_str |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
992 |
|> Type.constraint fT |> Syntax.check_term lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
993 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
994 |
val invariant_trm = Syntax.parse_term lthy invariant_str |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
995 |
|> Type.constraint ([domT, ranT] ---> @{typ bool}) |> Syntax.check_term lthy |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
996 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
997 |
val (globals, ctxt') = fix_globals domT ranT fvar lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
998 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
999 |
val Globals { x, h, ... } = globals |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1000 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1001 |
val clauses = map (mk_clause_context x ctxt') abstract_qglrs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1002 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1003 |
val n = length abstract_qglrs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1004 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1005 |
fun build_tree (ClauseContext { ctxt, rhs, ...}) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1006 |
Function_Ctx_Tree.mk_tree (fname, fT) h ctxt rhs |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1007 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1008 |
val trees = map build_tree clauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1009 |
val RCss = map find_calls trees |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1010 |
|
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
1011 |
val ((G, GIntro_thms, G_elim, G_induct), lthy) = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1012 |
PROFILE "def_graph" (define_graph (graph_name defname) fvar domT ranT clauses RCss) lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1013 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1014 |
val ((f, (_, f_defthm)), lthy) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1015 |
PROFILE "def_fun" (define_function (defname ^ "_sumC_def") (fname, mixfix) domT ranT G default) lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1016 |
|
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
1017 |
val RCss = map (map (inst_RC (Proof_Context.theory_of lthy) fvar f)) RCss |
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
1018 |
val trees = map (Function_Ctx_Tree.inst_tree (Proof_Context.theory_of lthy) fvar f) trees |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1019 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1020 |
val ((R, RIntro_thmss, R_elim), lthy) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1021 |
PROFILE "def_rel" (define_recursion_relation (rel_name defname) domT abstract_qglrs clauses RCss) lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1022 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1023 |
val (_, lthy) = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1024 |
Local_Theory.abbrev Syntax.mode_default ((Binding.name (dom_name defname), NoSyn), mk_acc domT R) lthy |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1025 |
|
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
1026 |
val newthy = Proof_Context.theory_of lthy |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1027 |
val clauses = map (transfer_clause_ctx newthy) clauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1028 |
|
3045
d0ad264f8c4f
updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Christian Urban <urbanc@in.tum.de>
parents:
2994
diff
changeset
|
1029 |
val cert = cterm_of (Proof_Context.theory_of lthy) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1030 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1031 |
val xclauses = PROFILE "xclauses" |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1032 |
(map7 (mk_clause_info globals G f) (1 upto n) clauses abstract_qglrs trees |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1033 |
RCss GIntro_thms) RIntro_thmss |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1034 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1035 |
val complete = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1036 |
mk_completeness globals clauses abstract_qglrs |> cert |> Thm.assume |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1037 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1038 |
val compat = |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
1039 |
mk_compat_proof_obligations domT ranT fvar f RCss invariant_trm abstract_qglrs |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1040 |
|> map (cert #> Thm.assume) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1041 |
|
2707
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
1042 |
val G_eqvt = mk_eqvt G |> cert |> Thm.assume |
747ebf2f066d
made eqvt-proof explicit in the function definitions
Christian Urban <urbanc@in.tum.de>
parents:
2677
diff
changeset
|
1043 |
|
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
1044 |
val invariant = mk_invariant globals G invariant_trm |> cert |> Thm.assume |
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
1045 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1046 |
val compat_store = store_compat_thms n compat |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1047 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1048 |
val (goalstate, values) = PROFILE "prove_stuff" |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1049 |
(prove_stuff lthy globals G f R xclauses complete compat |
2821
c7d4bd9e89e0
fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Christian Urban <urbanc@in.tum.de>
parents:
2819
diff
changeset
|
1050 |
compat_store G_elim G_eqvt invariant) f_defthm |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1051 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1052 |
fun mk_partial_rules provedgoal = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1053 |
let |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1054 |
val newthy = theory_of_thm provedgoal (*FIXME*) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1055 |
|
2974
b95a2065aa10
generated the partial eqvt-theorem for functions
Christian Urban <urbanc@in.tum.de>
parents:
2973
diff
changeset
|
1056 |
val ((graph_is_function, complete_thm), graph_is_eqvt) = |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1057 |
provedgoal |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1058 |
|> Conjunction.elim |
2974
b95a2065aa10
generated the partial eqvt-theorem for functions
Christian Urban <urbanc@in.tum.de>
parents:
2973
diff
changeset
|
1059 |
|>> fst o Conjunction.elim |
b95a2065aa10
generated the partial eqvt-theorem for functions
Christian Urban <urbanc@in.tum.de>
parents:
2973
diff
changeset
|
1060 |
|>> Conjunction.elim |
b95a2065aa10
generated the partial eqvt-theorem for functions
Christian Urban <urbanc@in.tum.de>
parents:
2973
diff
changeset
|
1061 |
|>> apfst (Thm.forall_elim_vars 0) |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1062 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1063 |
val f_iff = graph_is_function RS (f_defthm RS ex1_implies_iff) |
2974
b95a2065aa10
generated the partial eqvt-theorem for functions
Christian Urban <urbanc@in.tum.de>
parents:
2973
diff
changeset
|
1064 |
val f_eqvt = graph_is_function RS (graph_is_eqvt RS (f_defthm RS @{thm fundef_ex1_eqvt})) |
2973
d1038e67923a
added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents:
2885
diff
changeset
|
1065 |
|
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1066 |
val psimps = PROFILE "Proving simplification rules" |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1067 |
(mk_psimps newthy globals R xclauses values f_iff) graph_is_function |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1068 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1069 |
val simple_pinduct = PROFILE "Proving partial induction rule" |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1070 |
(mk_partial_induct_rule newthy globals R complete_thm) xclauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1071 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1072 |
val total_intro = PROFILE "Proving nested termination rule" |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1073 |
(mk_nest_term_rule newthy globals R R_elim) xclauses |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1074 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1075 |
val dom_intros = |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1076 |
if domintros then SOME (PROFILE "Proving domain introduction rules" |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1077 |
(map (mk_domain_intro lthy globals R R_elim)) xclauses) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1078 |
else NONE |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1079 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1080 |
in |
2973
d1038e67923a
added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents:
2885
diff
changeset
|
1081 |
NominalFunctionResult {fs=[f], G=G, R=R, cases=complete_thm, |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1082 |
psimps=psimps, simple_pinducts=[simple_pinduct], |
2973
d1038e67923a
added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Christian Urban <urbanc@in.tum.de>
parents:
2885
diff
changeset
|
1083 |
termination=total_intro, domintros=dom_intros, eqvts=[f_eqvt]} |
2665
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1084 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1085 |
in |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1086 |
((f, goalstate, mk_partial_rules), lthy) |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1087 |
end |
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1088 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1089 |
|
16b5a67ee279
exported nominal function code to external file
Christian Urban <urbanc@in.tum.de>
parents:
diff
changeset
|
1090 |
end |