| author | huffman |
| Thu, 14 Dec 2006 21:03:39 +0100 | |
| changeset 21850 | bf253f7075b4 |
| parent 21757 | 093ca3efb132 |
| child 21878 | cfc07819bb47 |
| permissions | -rw-r--r-- |
| 20319 | 1 |
(* |
2 |
ID: $Id$ |
|
3 |
Author: Amine Chaieb, TU Muenchen |
|
4 |
||
5 |
A trial for automatical reification. |
|
6 |
*) |
|
7 |
||
8 |
signature REFLECTION = sig |
|
9 |
val genreify_tac: Proof.context -> thm list -> term option -> int -> tactic |
|
10 |
val reflection_tac: Proof.context -> thm list -> term option -> int -> tactic |
|
11 |
end; |
|
12 |
||
13 |
structure Reflection : REFLECTION |
|
14 |
= struct |
|
15 |
||
| 20374 | 16 |
val ext2 = thm "ext2"; |
| 21669 | 17 |
val nth_Cons_0 = thm "nth_Cons_0"; |
18 |
val nth_Cons_Suc = thm "nth_Cons_Suc"; |
|
19 |
||
| 20374 | 20 |
(* Make a congruence rule out of a defining equation for the interpretation *) |
21 |
(* th is one defining equation of f, i.e. |
|
22 |
th is "f (Cp ?t1 ... ?tn) = P(f ?t1, .., f ?tn)" *) |
|
23 |
(* Cp is a constructor pattern and P is a pattern *) |
|
24 |
||
25 |
(* The result is: |
|
26 |
[|?A1 = f ?t1 ; .. ; ?An= f ?tn |] ==> P (?A1, .., ?An) = f (Cp ?t1 .. ?tn) *) |
|
27 |
(* + the a list of names of the A1 .. An, Those are fresh in the ctxt*) |
|
28 |
||
29 |
||
30 |
fun mk_congeq ctxt fs th = |
|
31 |
let |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
32 |
val (f as Const(fN,fT)) = th |> prop_of |> HOLogic.dest_Trueprop |> HOLogic.dest_eq |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
33 |
|> fst |> strip_comb |> fst |
| 20374 | 34 |
val thy = ProofContext.theory_of ctxt |
35 |
val cert = Thm.cterm_of thy |
|
36 |
val (((_,_),[th']), ctxt') = Variable.import true [th] ctxt |
|
37 |
val (lhs, rhs) = HOLogic.dest_eq (HOLogic.dest_Trueprop (Thm.prop_of th')) |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
38 |
fun add_fterms (t as t1 $ t2) = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
39 |
if exists (fn f => (t |> strip_comb |> fst) aconv f) fs then insert (op aconv) t |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
40 |
else add_fterms t1 #> add_fterms t2 |
| 20374 | 41 |
| add_fterms (t as Abs(xn,xT,t')) = |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
42 |
if (fN mem (term_consts t)) then (fn _ => [t]) else (fn _ => []) |
| 20374 | 43 |
| add_fterms _ = I |
44 |
val fterms = add_fterms rhs [] |
|
|
20797
c1f0bc7e7d80
renamed Variable.invent_fixes to Variable.variant_fixes;
wenzelm
parents:
20595
diff
changeset
|
45 |
val (xs, ctxt'') = Variable.variant_fixes (replicate (length fterms) "x") ctxt' |
| 20374 | 46 |
val tys = map fastype_of fterms |
47 |
val vs = map Free (xs ~~ tys) |
|
48 |
val env = fterms ~~ vs |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
49 |
(* FIXME!!!!*) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
50 |
fun replace_fterms (t as t1 $ t2) = |
| 20374 | 51 |
(case AList.lookup (op aconv) env t of |
52 |
SOME v => v |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
53 |
| NONE => replace_fterms t1 $ replace_fterms t2) |
| 20374 | 54 |
| replace_fterms t = (case AList.lookup (op aconv) env t of |
55 |
SOME v => v |
|
56 |
| NONE => t) |
|
57 |
||
58 |
fun mk_def (Abs(x,xT,t),v) = HOLogic.mk_Trueprop ((HOLogic.all_const xT)$ Abs(x,xT,HOLogic.mk_eq(v$(Bound 0), t))) |
|
59 |
| mk_def (t, v) = HOLogic.mk_Trueprop (HOLogic.mk_eq (v, t)) |
|
60 |
fun tryext x = (x RS ext2 handle _ => x) |
|
61 |
val cong = (Goal.prove ctxt'' [] (map mk_def env) |
|
62 |
(HOLogic.mk_Trueprop (HOLogic.mk_eq (lhs, replace_fterms rhs))) |
|
63 |
(fn x => LocalDefs.unfold_tac (#context x) (map tryext (#prems x)) |
|
64 |
THEN rtac th' 1)) RS sym |
|
65 |
||
66 |
val (cong' :: vars') = |
|
67 |
Variable.export ctxt'' ctxt (cong :: map (Drule.mk_term o cert) vs) |
|
68 |
val vs' = map (fst o fst o Term.dest_Var o Thm.term_of o Drule.dest_term) vars' |
|
69 |
||
70 |
in (vs', cong') end; |
|
| 20319 | 71 |
(* congs is a list of pairs (P,th) where th is a theorem for *) |
72 |
(* [| f p1 = A1; ...; f pn = An|] ==> f (C p1 .. pn) = P *) |
|
73 |
val FWD = curry (op OF); |
|
74 |
||
75 |
(* da is the decomposition for atoms, ie. it returns ([],g) where g |
|
76 |
returns the right instance f (AtC n) = t , where AtC is the Atoms |
|
77 |
constructor and n is the number of the atom corresponding to t *) |
|
78 |
||
79 |
(* Generic decomp for reification : matches the actual term with the |
|
80 |
rhs of one cong rule. The result of the matching guides the |
|
81 |
proof synthesis: The matches of the introduced Variables A1 .. An are |
|
82 |
processed recursively |
|
83 |
The rest is instantiated in the cong rule,i.e. no reification is needed *) |
|
84 |
||
| 20374 | 85 |
exception REIF of string; |
86 |
||
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
87 |
val bds = ref ([]: (typ * ((term list) * (term list))) list); |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
88 |
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
89 |
fun index_of t = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
90 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
91 |
val tt = HOLogic.listT (fastype_of t) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
92 |
in |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
93 |
(case AList.lookup (op =) (!bds) tt of |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
94 |
NONE => error "index_of : type not found in environements!" |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
95 |
| SOME (tbs,tats) => |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
96 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
97 |
val i = find_index_eq t tats |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
98 |
val j = find_index_eq t tbs |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
99 |
in (if j= ~1 then |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
100 |
if i= ~1 |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
101 |
then (bds := AList.update (op =) (tt,(tbs,tats@[t])) (!bds) ; |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
102 |
length tbs + length tats) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
103 |
else i else j) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
104 |
end) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
105 |
end; |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
106 |
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
107 |
fun dest_listT (Type ("List.list", [T])) = T;
|
| 20374 | 108 |
|
109 |
fun decomp_genreif da cgns (t,ctxt) = |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
110 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
111 |
val thy = ProofContext.theory_of ctxt |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
112 |
val cert = cterm_of thy |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
113 |
fun tryabsdecomp (s,ctxt) = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
114 |
(case s of |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
115 |
Abs(xn,xT,ta) => |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
116 |
(let |
|
20797
c1f0bc7e7d80
renamed Variable.invent_fixes to Variable.variant_fixes;
wenzelm
parents:
20595
diff
changeset
|
117 |
val ([xn],ctxt') = Variable.variant_fixes ["x"] ctxt |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
118 |
val (xn,ta) = variant_abs (xn,xT,ta) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
119 |
val x = Free(xn,xT) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
120 |
val _ = (case AList.lookup (op =) (!bds) (HOLogic.listT xT) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
121 |
of NONE => error "tryabsdecomp: Type not found in the Environement" |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
122 |
| SOME (bsT,atsT) => |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
123 |
(bds := AList.update (op =) (HOLogic.listT xT, ((x::bsT), atsT)) (!bds))) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
124 |
in ([(ta, ctxt')] , |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
125 |
fn [th] => ((let val (bsT,asT) = the(AList.lookup (op =) (!bds) (HOLogic.listT xT)) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
126 |
in (bds := AList.update (op =) (HOLogic.listT xT,(tl bsT,asT)) (!bds)) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
127 |
end) ; |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
128 |
hd (Variable.export ctxt' ctxt [(forall_intr (cert x) th) COMP allI]))) |
| 20374 | 129 |
end) |
130 |
| _ => da (s,ctxt)) |
|
131 |
in |
|
132 |
(case cgns of |
|
133 |
[] => tryabsdecomp (t,ctxt) |
|
134 |
| ((vns,cong)::congs) => ((let |
|
135 |
val cert = cterm_of thy |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
136 |
val certy = ctyp_of thy |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
137 |
val (tyenv, tmenv) = |
| 20319 | 138 |
Pattern.match thy |
139 |
((fst o HOLogic.dest_eq o HOLogic.dest_Trueprop) (concl_of cong), t) |
|
140 |
(Envir.type_env (Envir.empty 0),Term.Vartab.empty) |
|
141 |
val (fnvs,invs) = List.partition (fn ((vn,_),_) => vn mem vns) (Vartab.dest tmenv) |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
142 |
val (fts,its) = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
143 |
(map (snd o snd) fnvs, |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
144 |
map (fn ((vn,vi),(tT,t)) => (cert(Var ((vn,vi),tT)), cert t)) invs) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
145 |
val ctyenv = map (fn ((vn,vi),(s,ty)) => (certy (TVar((vn,vi),s)), certy ty)) (Vartab.dest tyenv) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
146 |
in (fts ~~ (replicate (length fts) ctxt), FWD (instantiate (ctyenv, its) cong)) |
| 20319 | 147 |
end) |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
148 |
handle MATCH => decomp_genreif da congs (t,ctxt))) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
149 |
end; |
| 20319 | 150 |
(* looks for the atoms equation and instantiates it with the right number *) |
| 20374 | 151 |
|
152 |
fun mk_decompatom eqs (t,ctxt) = |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
153 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
154 |
val tT = fastype_of t |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
155 |
fun isat eq = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
156 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
157 |
val rhs = eq |> prop_of |> HOLogic.dest_Trueprop |> HOLogic.dest_eq |> snd |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
158 |
in exists_Const |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
159 |
(fn (n,ty) => n="List.nth" |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
160 |
andalso |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
161 |
AList.defined (op =) (!bds) (domain_type ty)) rhs |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
162 |
andalso fastype_of rhs = tT |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
163 |
end |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
164 |
fun get_nth t = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
165 |
case t of |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
166 |
Const("List.nth",_)$vs$n => (t,vs,n)
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
167 |
| t1$t2 => (get_nth t1 handle REIF "get_nth" => get_nth t2) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
168 |
| Abs(_,_,t') => get_nth t' |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
169 |
| _ => raise REIF "get_nth" |
|
20797
c1f0bc7e7d80
renamed Variable.invent_fixes to Variable.variant_fixes;
wenzelm
parents:
20595
diff
changeset
|
170 |
val ([xn,vsn],ctxt') = Variable.variant_fixes ["x","vs"] ctxt |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
171 |
val thy = ProofContext.theory_of ctxt' |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
172 |
val cert = cterm_of thy |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
173 |
fun tryeqs [] = raise REIF "Can not find the atoms equation" |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
174 |
| tryeqs (eq::eqs) = (( |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
175 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
176 |
val rhs = eq |> prop_of |> HOLogic.dest_Trueprop |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
177 |
|> HOLogic.dest_eq |> snd |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
178 |
val (nt,vs,n) = get_nth rhs |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
179 |
val ntT = fastype_of nt |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
180 |
val ntlT = HOLogic.listT ntT |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
181 |
val (bsT,asT) = the (AList.lookup (op =) (!bds) ntlT) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
182 |
val x = Var ((xn,0),ntT) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
183 |
val rhs_P = subst_free [(nt,x)] rhs |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
184 |
val (_, tmenv) = Pattern.match |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
185 |
thy (rhs_P, t) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
186 |
(Envir.type_env (Envir.empty 0),Term.Vartab.empty) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
187 |
val tml = Vartab.dest tmenv |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
188 |
val SOME (_,t') = AList.lookup (op =) tml (xn,0) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
189 |
val cvs = |
| 21078 | 190 |
cert (fold_rev (fn x => fn xs => Const("List.list.Cons", ntT --> ntlT --> ntlT)$x$xs)
|
191 |
bsT (Free (vsn, ntlT))) |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
192 |
val cts = map (fn ((vn,vi),(tT,t)) => (cert(Var ((vn,vi),tT)), cert t)) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
193 |
(AList.delete (op =) (xn,0) tml) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
194 |
val th = (instantiate |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
195 |
([], |
| 21621 | 196 |
[(cert vs, cvs),(cert n, t' |> index_of |> IntInf.fromInt |> HOLogic.mk_nat |> cert)] |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
197 |
@cts) eq) RS sym |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
198 |
in hd (Variable.export ctxt' ctxt [th]) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
199 |
end) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
200 |
handle MATCH => tryeqs eqs) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
201 |
in ([], fn _ => tryeqs (filter isat eqs)) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
202 |
end; |
| 20374 | 203 |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
204 |
(* |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
205 |
fun mk_decompatom eqs (t,ctxt) = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
206 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
207 |
val tT = fastype_of t |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
208 |
val tlT = HOLogic.listT tT |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
209 |
val (bsT,asT) = (the (AList.lookup (op =) (!bds) tlT) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
210 |
handle Option => error "mk_decompatom: Type not found in the env.") |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
211 |
fun isateq (_$_$(Const("List.nth",_)$vs$_)) = (fastype_of vs = tlT)
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
212 |
| isateq _ = false |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
213 |
in case List.find (isateq o HOLogic.dest_Trueprop o prop_of) eqs of |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
214 |
NONE => raise REIF "Can not find the atoms equation" |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
215 |
| SOME th => |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
216 |
([], |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
217 |
fn ths => |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
218 |
let |
|
20797
c1f0bc7e7d80
renamed Variable.invent_fixes to Variable.variant_fixes;
wenzelm
parents:
20595
diff
changeset
|
219 |
val ([x], ctxt') = Variable.variant_fixes ["vs"] ctxt |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
220 |
val cert = cterm_of (ProofContext.theory_of ctxt') |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
221 |
val (Const("List.nth",_)$(vs as Var((vsn,vsi),_))$n) =
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
222 |
(snd o HOLogic.dest_eq o HOLogic.dest_Trueprop o prop_of) th |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
223 |
val cvs = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
224 |
cert (foldr (fn (x,xs) => Const("List.list.Cons", tT --> tlT --> tlT)$x$xs)
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
225 |
(Free(x,tlT)) bsT) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
226 |
val th' = (instantiate ([], |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
227 |
[(cert vs, cvs), |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
228 |
(cert n, cert (HOLogic.mk_nat(index_of t)))]) th) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
229 |
RS sym |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
230 |
in hd (Variable.export ctxt' ctxt [th']) end) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
231 |
end; |
| 20374 | 232 |
*) |
| 20319 | 233 |
(* Generic reification procedure: *) |
234 |
(* creates all needed cong rules and then just uses the theorem synthesis *) |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
235 |
|
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
236 |
fun mk_congs ctxt raw_eqs = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
237 |
let |
| 21078 | 238 |
val fs = fold_rev (fn eq => |
| 20853 | 239 |
insert (op =) (eq |> prop_of |> HOLogic.dest_Trueprop |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
240 |
|> HOLogic.dest_eq |> fst |> strip_comb |
| 21078 | 241 |
|> fst)) raw_eqs [] |
242 |
val tys = fold_rev (fn f => fn ts => (f |> fastype_of |> binder_types |> split_last |> fst) |
|
243 |
union ts) fs [] |
|
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
244 |
val _ = bds := AList.make (fn _ => ([],[])) tys |
|
20797
c1f0bc7e7d80
renamed Variable.invent_fixes to Variable.variant_fixes;
wenzelm
parents:
20595
diff
changeset
|
245 |
val (vs, ctxt') = Variable.variant_fixes (replicate (length tys) "vs") ctxt |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
246 |
val thy = ProofContext.theory_of ctxt' |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
247 |
val cert = cterm_of thy |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
248 |
val vstys = map (fn (t,v) => (t,SOME (cert (Free(v,t))))) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
249 |
(tys ~~ vs) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
250 |
fun insteq eq ts = |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
251 |
let val itms = map (fn t => t|> (AList.lookup (op =) vstys) |> the) ts |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
252 |
in instantiate' [] itms eq |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
253 |
end |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
254 |
val eqs = map (fn eq => eq |> prop_of |> HOLogic.dest_Trueprop |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
255 |
|> HOLogic.dest_eq |> fst |> strip_comb |> fst |> fastype_of |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
256 |
|> binder_types |> split_last |> fst |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
257 |
|> (insteq eq)) raw_eqs |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
258 |
val (ps,congs) = split_list (map (mk_congeq ctxt' fs) eqs) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
259 |
in ps ~~ (Variable.export ctxt' ctxt congs) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
260 |
end; |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
261 |
|
| 20319 | 262 |
fun genreif ctxt raw_eqs t = |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
263 |
let |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
264 |
val _ = bds := [] |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
265 |
val congs = mk_congs ctxt raw_eqs |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
266 |
val th = divide_and_conquer (decomp_genreif (mk_decompatom raw_eqs) congs) (t,ctxt) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
267 |
val tys = th |> prop_of |> HOLogic.dest_Trueprop |> HOLogic.dest_eq |> snd |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
268 |
|> strip_comb |> fst |> fastype_of |> strip_type |> fst |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
269 |
|> split_last |> fst |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
270 |
val cert = cterm_of (ProofContext.theory_of ctxt) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
271 |
val cvs = map (fn t => t |> (AList.lookup (op =) (!bds)) |> the |> snd |
| 21757 | 272 |
|> HOLogic.mk_list (dest_listT t) |> cert |> SOME) |
|
20564
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
273 |
tys |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
274 |
val th' = (instantiate' [] cvs (th RS sym)) RS sym |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
275 |
val t' = (fst o HOLogic.dest_eq o HOLogic.dest_Trueprop o prop_of) th' |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
276 |
val th'' = Goal.prove ctxt [] [] (HOLogic.mk_Trueprop (HOLogic.mk_eq (t, t'))) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
277 |
(fn _ => Simp_tac 1) |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
278 |
val _ = bds := [] |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
279 |
in FWD trans [th'',th'] |
|
6857bd9f1a79
Reifiaction now deals with Interpretations with an arbtrary number of parameters. It deals with binding. The Atomic cases can be I ... = f (xs!n)
chaieb
parents:
20374
diff
changeset
|
280 |
end; |
| 20319 | 281 |
|
282 |
fun genreflect ctxt corr_thm raw_eqs t = |
|
283 |
let val th = FWD trans [genreif ctxt raw_eqs t, corr_thm RS sym] |
|
284 |
val ft = (snd o Thm.dest_comb o snd o Thm.dest_comb o snd o Thm.dest_comb o cprop_of) th |
|
| 20595 | 285 |
val rth = NBE.normalization_conv ft |
| 20319 | 286 |
in simplify (HOL_basic_ss addsimps raw_eqs addsimps [nth_Cons_0, nth_Cons_Suc]) |
287 |
(simplify (HOL_basic_ss addsimps [rth]) th) |
|
288 |
end |
|
289 |
||
290 |
fun genreify_tac ctxt eqs to i = (fn st => |
|
291 |
let |
|
292 |
val P = HOLogic.dest_Trueprop (List.nth (prems_of st, i - 1)) |
|
293 |
val t = (case to of NONE => P | SOME x => x) |
|
294 |
val th = (genreif ctxt eqs t) RS ssubst |
|
295 |
in rtac th i st |
|
296 |
end); |
|
297 |
||
298 |
(* Reflection calls reification and uses the correctness *) |
|
299 |
(* theorem assumed to be the dead of the list *) |
|
300 |
fun reflection_tac ctxt (corr_thm::raw_eqs) to i = |
|
301 |
(fn st => |
|
302 |
let val P = (HOLogic.dest_Trueprop (List.nth (prems_of st, i - 1))) |
|
303 |
val t = (case to of NONE => P | SOME x => x) |
|
304 |
val th = (genreflect ctxt corr_thm raw_eqs t) RS ssubst |
|
305 |
in rtac th i st end); |
|
306 |
||
|
20797
c1f0bc7e7d80
renamed Variable.invent_fixes to Variable.variant_fixes;
wenzelm
parents:
20595
diff
changeset
|
307 |
end |