| author | wenzelm | 
| Sat, 07 Oct 2006 01:31:01 +0200 | |
| changeset 20873 | 4066ee15b278 | 
| parent 20305 | 16c8f44b1852 | 
| child 20893 | c99f79910ae8 | 
| permissions | -rw-r--r-- | 
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 1 | (* Title: Pure/Tools/invoke.ML | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 2 | ID: $Id$ | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 3 | Author: Makarius | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 4 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 5 | Schematic invocation of locale expression in proof context. | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 6 | *) | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 7 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 8 | signature INVOKE = | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 9 | sig | 
| 19849 | 10 | val invoke: string * Attrib.src list -> Locale.expr -> string option list -> | 
| 11 | (string * string option * mixfix) list -> bool -> Proof.state -> Proof.state | |
| 12 | val invoke_i: string * attribute list -> Locale.expr -> term option list -> | |
| 13 | (string * typ option * mixfix) list -> bool -> Proof.state -> Proof.state | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 14 | end; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 15 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 16 | structure Invoke: INVOKE = | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 17 | struct | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 18 | |
| 19849 | 19 | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 20 | (* invoke *) | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 21 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 22 | local | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 23 | |
| 19849 | 24 | fun gen_invoke prep_att prep_expr prep_terms add_fixes | 
| 25 | (prfx, raw_atts) raw_expr raw_insts fixes int state = | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 26 | let | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 27 | val _ = Proof.assert_forward_or_chain state; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 28 | val thy = Proof.theory_of state; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 29 | |
| 19849 | 30 | val more_atts = map (prep_att thy) raw_atts; | 
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 31 | val (elems, _) = prep_expr raw_expr [] (ProofContext.init thy); | 
| 19849 | 32 | |
| 33 | val prems = maps Element.prems_of elems; | |
| 34 | val params = maps Element.params_of elems; | |
| 35 | val types = rev (fold Term.add_tfrees prems (fold (Term.add_tfreesT o #2) params [])); | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 36 | |
| 19849 | 37 | val prems' = map Logic.varify prems; | 
| 38 | val params' = map (Logic.varify o Free) params; | |
| 39 | val types' = map (Logic.varifyT o TFree) types; | |
| 40 | ||
| 41 | val state' = state | |
| 42 | |> Proof.begin_block | |
| 43 | |> Proof.map_context (snd o add_fixes fixes); | |
| 44 | val ctxt' = Proof.context_of state'; | |
| 45 | ||
| 46 | val raw_insts' = zip_options params' raw_insts | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 47 | handle Library.UnequalLengths => error "Too many instantiations"; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 48 | val insts = map #1 raw_insts' ~~ | 
| 19849 | 49 | prep_terms ctxt' (map (fn (t, u) => (u, Term.fastype_of t)) raw_insts'); | 
| 50 | val inst_rules = | |
| 51 | replicate (length types') Drule.termI @ | |
| 52 | map (fn t => | |
| 53 | (case AList.lookup (op =) insts t of | |
| 54 | SOME u => Drule.mk_term (Thm.cterm_of thy u) | |
| 55 | | NONE => Drule.termI)) params'; | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 56 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 57 | val propp = | 
| 19849 | 58 |       [(("", []), map (rpair [] o Logic.mk_term o Logic.mk_type) types'),
 | 
| 59 |        (("", []), map (rpair [] o Logic.mk_term) params'),
 | |
| 60 |        (("", []), map (rpair [] o Element.mark_witness) prems')];
 | |
| 61 | fun after_qed results = | |
| 62 | Proof.end_block #> | |
| 20305 | 63 | Proof.map_context (fn ctxt => | 
| 19849 | 64 | let | 
| 65 | val ([res_types, res_params, res_prems], ctxt'') = | |
| 20218 
be3bfb0699ba
Variable.import(T): result includes fixed types/terms;
 wenzelm parents: 
19919diff
changeset | 66 | fold_burrow (apfst snd oo Variable.import false) results ctxt'; | 
| 19849 | 67 | |
| 68 | val types'' = map (Logic.dest_type o Thm.term_of o Drule.dest_term) res_types; | |
| 69 | val params'' = map (Thm.term_of o Drule.dest_term) res_params; | |
| 70 | val elems' = elems |> map (Element.inst_ctxt thy | |
| 71 | (Symtab.make (map #1 types ~~ types''), Symtab.make (map #1 params ~~ params''))); | |
| 19868 | 72 | val prems'' = map2 Element.make_witness (maps Element.prems_of elems') res_prems; | 
| 20266 | 73 | val notes = | 
| 74 | maps (Element.facts_of thy) elems' | |
| 75 | |> Element.satisfy_facts prems'' | |
| 76 | |> Element.generalize_facts ctxt'' ctxt | |
| 19849 | 77 | |> Attrib.map_facts (Attrib.attribute_i thy) | 
| 20266 | 78 | |> map (fn ((a, atts), bs) => ((a, atts @ more_atts), bs)); | 
| 19849 | 79 | in | 
| 80 | ctxt | |
| 81 | |> ProofContext.sticky_prefix prfx | |
| 82 | |> ProofContext.qualified_names | |
| 20266 | 83 | |> (snd o ProofContext.note_thmss_i notes) | 
| 19849 | 84 | |> ProofContext.restore_naming ctxt | 
| 20305 | 85 | end) #> | 
| 86 | Proof.put_facts NONE #> Seq.single; | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 87 | in | 
| 19849 | 88 | state' | 
| 19868 | 89 | |> Proof.local_goal (K (K ())) (K I) ProofContext.bind_propp_schematic_i | 
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 90 | "invoke" NONE after_qed propp | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 91 | |> Element.refine_witness | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 92 | |> Seq.hd | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 93 | |> Proof.refine (Method.Basic (K (Method.METHOD (K (HEADGOAL (RANGE (map rtac inst_rules))))))) | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 94 | |> Seq.hd | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 95 | end; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 96 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 97 | (* FIXME *) | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 98 | fun read_terms ctxt args = | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 99 | #1 (ProofContext.read_termTs ctxt (K false) (K NONE) (K NONE) [] args) | 
| 19897 
fe661eb3b0e7
ProofContext: moved variable operations to struct Variable;
 wenzelm parents: 
19868diff
changeset | 100 | |> Variable.polymorphic ctxt; | 
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 101 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 102 | (* FIXME *) | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 103 | fun cert_terms ctxt args = map fst args; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 104 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 105 | in | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 106 | |
| 19849 | 107 | fun invoke x = gen_invoke Attrib.attribute Locale.read_expr read_terms ProofContext.add_fixes x; | 
| 108 | fun invoke_i x = gen_invoke (K I) Locale.cert_expr cert_terms ProofContext.add_fixes_i x; | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 109 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 110 | end; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 111 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 112 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 113 | (* concrete syntax *) | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 114 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 115 | local structure P = OuterParse and K = OuterKeyword in | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 116 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 117 | val invokeP = | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 118 | OuterSyntax.command "invoke" | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 119 | "schematic invocation of locale expression in proof context" | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 120 | (K.tag_proof K.prf_goal) | 
| 19849 | 121 | (P.opt_thm_name ":" -- P.locale_expr -- P.locale_insts -- P.for_fixes | 
| 122 | >> (fn (((name, expr), insts), fixes) => | |
| 123 | Toplevel.print o Toplevel.proof' (invoke name expr insts fixes))); | |
| 19813 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 124 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 125 | val _ = OuterSyntax.add_parsers [invokeP]; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 126 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 127 | end; | 
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 128 | |
| 
b051be997d50
Schematic invocation of locale expression in proof context.
 wenzelm parents: diff
changeset | 129 | end; |