src/Pure/Isar/obtain.ML
author wenzelm
Mon, 03 Jul 2006 19:33:09 +0200
changeset 19978 df19a7876183
parent 19906 c23a0e65b285
child 20004 e6d3f2b031e6
permissions -rw-r--r--
obtain_export: Thm.generalize; guess: fixed handling of mixfixes of vars; tuned;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/Isar/obtain.ML
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
     3
    Author:     Markus Wenzel, TU Muenchen
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
     4
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
     5
The 'obtain' and 'guess' language elements -- generalized existence at
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
     6
the level of proof texts: 'obtain' involves a proof that certain
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
     7
fixes/assumes may be introduced into the present context; 'guess' is
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
     8
similar, but derives these elements from the course of reasoning!
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
     9
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    10
  <chain_facts>
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    11
  obtain x where "A x" <proof> ==
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    12
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    13
  have "!!thesis. (!!x. A x ==> thesis) ==> thesis"
12970
c9b1838a2cc0 improved messages;
wenzelm
parents: 12404
diff changeset
    14
  proof succeed
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    15
    fix thesis
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    16
    assume that [intro?]: "!!x. A x ==> thesis"
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    17
    <chain_facts>
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    18
    show thesis
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    19
      apply (insert that)
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    20
      <proof>
12970
c9b1838a2cc0 improved messages;
wenzelm
parents: 12404
diff changeset
    21
  qed
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    22
  fix x assm <<obtain_export>> "A x"
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    23
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    24
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    25
  <chain_facts>
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    26
  guess x <proof body> <proof end> ==
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    27
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    28
  {
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    29
    fix thesis
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    30
    <chain_facts> have "PROP ?guess"
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    31
      apply magic      -- {* turns goal into "thesis ==> #thesis" *}
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    32
      <proof body>
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    33
      apply_end magic  -- {* turns final "(!!x. P x ==> thesis) ==> #thesis" into
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    34
        "#((!!x. A x ==> thesis) ==> thesis)" which is a finished goal state *}
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    35
      <proof end>
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    36
  }
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    37
  fix x assm <<obtain_export>> "A x"
8094
62b45a2e6ecb ObtainFun;
wenzelm
parents: 7923
diff changeset
    38
*)
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    39
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    40
signature OBTAIN =
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    41
sig
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
    42
  val obtain: string -> (string * string option * mixfix) list ->
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
    43
    ((string * Attrib.src list) * (string * string list) list) list
17357
ee2bdca144c7 tuned Isar proof elements;
wenzelm
parents: 17111
diff changeset
    44
    -> bool -> Proof.state -> Proof.state
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
    45
  val obtain_i: string -> (string * typ option * mixfix) list ->
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
    46
    ((string * attribute list) * (term * term list) list) list
17357
ee2bdca144c7 tuned Isar proof elements;
wenzelm
parents: 17111
diff changeset
    47
    -> bool -> Proof.state -> Proof.state
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
    48
  val guess: (string * string option * mixfix) list -> bool -> Proof.state -> Proof.state
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
    49
  val guess_i: (string * typ option * mixfix) list -> bool -> Proof.state -> Proof.state
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    50
  val statement: (string * ((string * 'typ option) list * 'term list)) list ->
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    51
    (('typ, 'term, 'fact) Element.ctxt list *
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
    52
      ((string * Attrib.src list) * ('term * 'term list) list) list) *
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
    53
    (((string * Attrib.src list) * (term * term list) list) list -> Proof.context ->
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
    54
      (((string * Attrib.src list) * (term * term list) list) list * thm list) * Proof.context)
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    55
end;
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    56
10379
93630e0c5ae9 improved handling of "that": insert into goal, only declare as Pure "intro";
wenzelm
parents: 9481
diff changeset
    57
structure Obtain: OBTAIN =
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    58
struct
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
    59
8094
62b45a2e6ecb ObtainFun;
wenzelm
parents: 7923
diff changeset
    60
18670
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
    61
(** obtain_export **)
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
    62
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    63
(*
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    64
  [x, A x]
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    65
     :
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    66
     B
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    67
  --------
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    68
     B
18870
020e242c02a0 tuned comments;
wenzelm
parents: 18769
diff changeset
    69
*)
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
    70
fun obtain_export ctxt parms rule cprops thm =
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    71
  let
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    72
    val {thy, prop, ...} = Thm.rep_thm thm;
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    73
    val concl = Logic.strip_assums_concl prop;
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    74
    val bads = Term.fold_aterms (fn v as Free (x, _) =>
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    75
      if member (op =) parms x then insert (op aconv) v else I | _ => I) concl [];
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    76
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    77
    val thm' = thm |> Drule.implies_intr_protected cprops;
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    78
    val thm'' = thm' |> Thm.generalize ([], parms) (Thm.maxidx_of thm' + 1);
18040
c67505cdecad renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17974
diff changeset
    79
    val elim_tacs = replicate (length cprops) (Tactic.etac Drule.protectI);
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    80
  in
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    81
    if not (null bads) then
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
    82
      error ("Conclusion contains obtained parameters: " ^
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
    83
        space_implode " " (map (ProofContext.string_of_term ctxt) bads))
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    84
    else if not (ObjectLogic.is_judgment thy concl) then
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    85
      error "Conclusion in obtained context must be object-logic judgment"
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
    86
    else (Tactic.rtac thm'' THEN' RANGE elim_tacs) 1 rule
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    87
  end;
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    88
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    89
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
    90
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    91
(** obtain **)
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    92
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    93
fun bind_judgment ctxt name =
18670
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
    94
  let
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
    95
    val (bind, _) = ProofContext.bind_fixes [name] ctxt;
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
    96
    val (t as _ $ Free v) = bind (ObjectLogic.fixed_judgment (ProofContext.theory_of ctxt) name);
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    97
  in (v, t) end;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
    98
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
    99
val thatN = "that";
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   100
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   101
local
8094
62b45a2e6ecb ObtainFun;
wenzelm
parents: 7923
diff changeset
   102
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   103
fun gen_obtain prep_att prep_vars prep_propp
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   104
    name raw_vars raw_asms int state =
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   105
  let
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
   106
    val _ = Proof.assert_forward_or_chain state;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   107
    val ctxt = Proof.context_of state;
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   108
    val thy = Proof.theory_of state;
17357
ee2bdca144c7 tuned Isar proof elements;
wenzelm
parents: 17111
diff changeset
   109
    val chain_facts = if can Proof.assert_chain state then Proof.the_facts state else [];
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   110
8543
f54926bded7b handle general case: params and hyps of thesis;
wenzelm
parents: 8109
diff changeset
   111
    (*obtain vars*)
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
   112
    val (vars, vars_ctxt) = prep_vars raw_vars ctxt;
18670
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
   113
    val (_, fix_ctxt) = vars_ctxt |> ProofContext.add_fixes_i vars;
c3f445b92aff uniform handling of fixes;
wenzelm
parents: 18643
diff changeset
   114
    val xs = map #1 vars;
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   115
8543
f54926bded7b handle general case: params and hyps of thesis;
wenzelm
parents: 8109
diff changeset
   116
    (*obtain asms*)
11890
28e42a90bea8 improved source arrangement of obtain;
wenzelm
parents: 11816
diff changeset
   117
    val (asms_ctxt, proppss) = prep_propp (fix_ctxt, map snd raw_asms);
19482
9f11af8f7ef9 tuned basic list operators (flat, maps, map_filter);
wenzelm
parents: 19300
diff changeset
   118
    val asm_props = maps (map fst) proppss;
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   119
    val asms = map fst (Attrib.map_specs (prep_att thy) raw_asms) ~~ proppss;
10464
b7b916a82dca tuned statement args;
wenzelm
parents: 10379
diff changeset
   120
19897
fe661eb3b0e7 ProofContext: moved variable operations to struct Variable;
wenzelm
parents: 19844
diff changeset
   121
    val _ = Variable.warn_extra_tfrees fix_ctxt asms_ctxt;
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   122
12970
c9b1838a2cc0 improved messages;
wenzelm
parents: 12404
diff changeset
   123
    (*obtain statements*)
16606
e45c9a95a554 no Syntax.internal on thesis;
wenzelm
parents: 15570
diff changeset
   124
    val thesisN = Term.variant xs AutoBind.thesisN;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   125
    val (thesis_var, thesis) = bind_judgment fix_ctxt thesisN;
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
   126
10582
49ebade930ea fixed binding of parameters;
wenzelm
parents: 10464
diff changeset
   127
    fun occs_var x = Library.get_first (fn t =>
18151
32538cf750ca guess: Seq.hd;
wenzelm
parents: 18124
diff changeset
   128
      Term.find_free t (ProofContext.get_skolem fix_ctxt x)) asm_props;
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   129
    val parms =
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   130
      map_filter (fn (SOME (Free a), x) => SOME (a, x) | _ => NONE) (map occs_var xs ~~ xs);
10582
49ebade930ea fixed binding of parameters;
wenzelm
parents: 10464
diff changeset
   131
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   132
    val that_name = if name = "" then thatN else name;
10582
49ebade930ea fixed binding of parameters;
wenzelm
parents: 10464
diff changeset
   133
    val that_prop =
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   134
      Term.list_all_free (map #1 parms, Logic.list_implies (asm_props, thesis))
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   135
      |> Library.curry Logic.list_rename_params (map #2 parms);
12970
c9b1838a2cc0 improved messages;
wenzelm
parents: 12404
diff changeset
   136
    val obtain_prop =
c9b1838a2cc0 improved messages;
wenzelm
parents: 12404
diff changeset
   137
      Logic.list_rename_params ([AutoBind.thesisN],
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   138
        Term.list_all_free ([thesis_var], Logic.mk_implies (that_prop, thesis)));
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   139
18124
a310c78298f9 simplified after_qed;
wenzelm
parents: 18040
diff changeset
   140
    fun after_qed _ =
17357
ee2bdca144c7 tuned Isar proof elements;
wenzelm
parents: 17111
diff changeset
   141
      Proof.local_qed (NONE, false)
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   142
      #> Seq.map (`Proof.the_fact #-> (fn rule =>
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
   143
        Proof.fix_i (map2 (fn x => fn (_, T, mx) => (x, T, mx)) xs vars)
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   144
        #> Proof.assm_i (K (obtain_export ctxt (map (#1 o #1) parms) rule)) asms));
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   145
  in
8094
62b45a2e6ecb ObtainFun;
wenzelm
parents: 7923
diff changeset
   146
    state
9468
9adbcf6375c1 turned into plain context element;
wenzelm
parents: 9293
diff changeset
   147
    |> Proof.enter_forward
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   148
    |> Proof.have_i NONE (K Seq.single) [(("", []), [(obtain_prop, [])])] int
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   149
    |> Proof.proof (SOME Method.succeed_text) |> Seq.hd
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
   150
    |> Proof.fix_i [(thesisN, NONE, NoSyn)]
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   151
    |> Proof.assume_i [((that_name, [ContextRules.intro_query NONE]), [(that_prop, [])])]
16842
wenzelm
parents: 16787
diff changeset
   152
    |> `Proof.the_facts
17357
ee2bdca144c7 tuned Isar proof elements;
wenzelm
parents: 17111
diff changeset
   153
    ||> Proof.chain_facts chain_facts
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   154
    ||> Proof.show_i NONE after_qed [(("", []), [(thesis, [])])] false
18907
f984f22f1cb4 Proof.refine_insert;
wenzelm
parents: 18897
diff changeset
   155
    |-> Proof.refine_insert
7674
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   156
  end;
99305245f6bd The 'obtain' language element -- achieves (eliminated) existential
wenzelm
parents:
diff changeset
   157
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   158
in
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   159
18728
6790126ab5f6 simplified type attribute;
wenzelm
parents: 18693
diff changeset
   160
val obtain = gen_obtain Attrib.attribute ProofContext.read_vars ProofContext.read_propp;
17111
d2ea9c974570 prepare attributes here;
wenzelm
parents: 17034
diff changeset
   161
val obtain_i = gen_obtain (K I) ProofContext.cert_vars ProofContext.cert_propp;
8094
62b45a2e6ecb ObtainFun;
wenzelm
parents: 7923
diff changeset
   162
62b45a2e6ecb ObtainFun;
wenzelm
parents: 7923
diff changeset
   163
end;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   164
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   165
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   166
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   167
(** guess **)
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   168
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   169
local
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   170
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   171
fun unify_params vars thesis_name raw_rule ctxt =
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   172
  let
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   173
    val thy = ProofContext.theory_of ctxt;
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   174
    val certT = Thm.ctyp_of thy;
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   175
    val cert = Thm.cterm_of thy;
17891
7a6c4d60a913 tuned error msg;
wenzelm
parents: 17858
diff changeset
   176
    val string_of_typ = ProofContext.string_of_typ ctxt;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   177
    val string_of_term = setmp show_types true (ProofContext.string_of_term ctxt);
17891
7a6c4d60a913 tuned error msg;
wenzelm
parents: 17858
diff changeset
   178
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   179
    fun err msg th = error (msg ^ ":\n" ^ ProofContext.string_of_thm ctxt th);
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   180
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   181
    val maxidx = fold (Term.maxidx_typ o snd o fst) vars ~1;
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   182
    val rule = Thm.incr_indexes (maxidx + 1) raw_rule;
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   183
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   184
    val params = RuleCases.strip_params (Logic.nth_prem (1, Thm.prop_of rule));
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   185
    val m = length vars;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   186
    val n = length params;
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   187
    val _ = m <= n orelse err "More variables than parameters in obtained rule" rule;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   188
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   189
    fun unify ((x, T), (y, U)) (tyenv, max) = Sign.typ_unify thy (T, U) (tyenv, max)
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   190
      handle Type.TUNIFY =>
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   191
        err ("Failed to unify variable " ^
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   192
          string_of_term (Free (x, Envir.norm_type tyenv T)) ^ " against parameter " ^
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   193
          string_of_term (Syntax.mark_boundT (y, Envir.norm_type tyenv U)) ^ " in") rule;
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   194
    val (tyenv, _) = fold unify (map #1 vars ~~ Library.take (m, params))
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   195
      (Vartab.empty, Int.max (maxidx, Thm.maxidx_of rule));
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   196
    val norm_type = Envir.norm_type tyenv;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   197
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   198
    val xs = map (apsnd norm_type o fst) vars;
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   199
    val ys = map (apsnd norm_type) (Library.drop (m, params));
19906
c23a0e65b285 Term.internal;
wenzelm
parents: 19897
diff changeset
   200
    val ys' = map Term.internal (Term.variantlist (map fst ys, map fst xs)) ~~ map #2 ys;
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   201
    val terms = map (Drule.mk_term o cert o Free) (xs @ ys');
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   202
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   203
    val instT =
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   204
      fold (Term.add_tvarsT o #2) params []
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   205
      |> map (TVar #> (fn T => (certT T, certT (norm_type T))));
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   206
    val (rule' :: terms', ctxt') =
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   207
      Variable.import false (Thm.instantiate (instT, []) rule :: terms) ctxt;
17891
7a6c4d60a913 tuned error msg;
wenzelm
parents: 17858
diff changeset
   208
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   209
    val vars' =
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   210
      map (dest_Free o Thm.term_of o Drule.dest_term) terms' ~~
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   211
      (map snd vars @ replicate (length ys) NoSyn);
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   212
    val rule'' = Thm.generalize ([], [thesis_name]) (Thm.maxidx_of rule' + 1) rule';
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   213
  in ((vars', rule''), ctxt') end;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   214
18693
8ae076ee5e19 guess: used fixed inferred_type of vars;
wenzelm
parents: 18678
diff changeset
   215
fun inferred_type (x, _, mx) ctxt =
18769
e90eb0bc0ddd ProofContext.inferred_param;
wenzelm
parents: 18728
diff changeset
   216
  let val ((_, T), ctxt') = ProofContext.inferred_param x ctxt
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   217
  in ((x, T, mx), ctxt') end;
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   218
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   219
fun polymorphic (vars, ctxt) =
19897
fe661eb3b0e7 ProofContext: moved variable operations to struct Variable;
wenzelm
parents: 19844
diff changeset
   220
  let val Ts = map Logic.dest_type (Variable.polymorphic ctxt (map (Logic.mk_type o #2) vars))
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   221
  in map2 (fn (x, _, mx) => fn T => ((x, T), mx)) vars Ts end;
18693
8ae076ee5e19 guess: used fixed inferred_type of vars;
wenzelm
parents: 18678
diff changeset
   222
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   223
fun gen_guess prep_vars raw_vars int state =
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   224
  let
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   225
    val _ = Proof.assert_forward_or_chain state;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   226
    val thy = Proof.theory_of state;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   227
    val ctxt = Proof.context_of state;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   228
    val chain_facts = if can Proof.assert_chain state then Proof.the_facts state else [];
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   229
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   230
    val ((thesis_name, _), thesis) = bind_judgment ctxt AutoBind.thesisN;
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
   231
    val vars = ctxt |> prep_vars raw_vars |-> fold_map inferred_type |> polymorphic;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   232
17974
5b54db4a44ee improved check_result;
wenzelm
parents: 17891
diff changeset
   233
    fun check_result th =
5b54db4a44ee improved check_result;
wenzelm
parents: 17891
diff changeset
   234
      (case Thm.prems_of th of
5b54db4a44ee improved check_result;
wenzelm
parents: 17891
diff changeset
   235
        [prem] =>
5b54db4a44ee improved check_result;
wenzelm
parents: 17891
diff changeset
   236
          if Thm.concl_of th aconv thesis andalso
5b54db4a44ee improved check_result;
wenzelm
parents: 17891
diff changeset
   237
            Logic.strip_assums_concl prem aconv thesis then ()
18678
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   238
          else error ("Guessed a different clause:\n" ^ ProofContext.string_of_thm ctxt th)
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   239
      | [] => error "Goal solved -- nothing guessed."
dd0c569fa43d sane ERROR handling;
wenzelm
parents: 18670
diff changeset
   240
      | _ => error ("Guess split into several cases:\n" ^ ProofContext.string_of_thm ctxt th));
17891
7a6c4d60a913 tuned error msg;
wenzelm
parents: 17858
diff changeset
   241
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   242
    fun guess_context raw_rule state' =
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   243
      let
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   244
        val ((parms, rule), ctxt') =
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   245
          unify_params vars thesis_name raw_rule (Proof.context_of state');
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   246
        val (bind, _) = ProofContext.bind_fixes (map (#1 o #1) parms) ctxt';
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   247
        val ts = map (bind o Free o #1) parms;
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   248
        val ps = map dest_Free ts;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   249
        val asms =
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   250
          Logic.strip_assums_hyp (Logic.nth_prem (1, Thm.prop_of rule))
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   251
          |> map (fn asm => (Term.betapplys (Term.list_abs (ps, asm), ts), []));
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   252
        val _ = not (null asms) orelse error "Trivial result -- nothing guessed";
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   253
      in
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   254
        state'
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   255
        |> Proof.map_context (K ctxt')
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   256
        |> Proof.fix_i (map (fn ((x, T), mx) => (x, SOME T, mx)) parms)
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   257
        |> Proof.assm_i (K (obtain_export ctxt' (map #1 ps) rule)) [(("", []), asms)]
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   258
        |> Proof.add_binds_i AutoBind.no_facts
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   259
      end;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   260
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   261
    val goal = Var (("guess", 0), propT);
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   262
    fun print_result ctxt' (k, [(s, [_, th])]) =
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   263
      ProofDisplay.print_results int ctxt' (k, [(s, [th])]);
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   264
    val before_qed = SOME (Method.primitive_text (Goal.conclude #> (fn th =>
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   265
      Goal.protect (Conjunction.intr (Drule.mk_term (Thm.cprop_of th)) th))));
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   266
    fun after_qed [[_, res]] =
19978
df19a7876183 obtain_export: Thm.generalize;
wenzelm
parents: 19906
diff changeset
   267
      (check_result res; Proof.end_block #> Seq.map (guess_context res));
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   268
  in
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   269
    state
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   270
    |> Proof.enter_forward
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   271
    |> Proof.begin_block
19844
2c1fdc397ded fixes: include mixfix syntax;
wenzelm
parents: 19779
diff changeset
   272
    |> Proof.fix_i [(AutoBind.thesisN, NONE, NoSyn)]
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   273
    |> Proof.chain_facts chain_facts
19779
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   274
    |> Proof.local_goal print_result (K I) (apsnd (rpair I))
5c77dfb74c7b guess: more careful about local polymorphism;
wenzelm
parents: 19585
diff changeset
   275
      "guess" before_qed after_qed [(("", []), [Logic.mk_term goal, goal])]
18151
32538cf750ca guess: Seq.hd;
wenzelm
parents: 18124
diff changeset
   276
    |> Proof.refine (Method.primitive_text (K (Goal.init (Thm.cterm_of thy thesis)))) |> Seq.hd
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   277
  end;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   278
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   279
in
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   280
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   281
val guess = gen_guess ProofContext.read_vars;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   282
val guess_i = gen_guess ProofContext.cert_vars;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   283
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   284
end;
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   285
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   286
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   287
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   288
(** statements with several cases **)
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   289
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   290
fun statement cases =
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   291
  let
18907
f984f22f1cb4 Proof.refine_insert;
wenzelm
parents: 18897
diff changeset
   292
    val names =
f984f22f1cb4 Proof.refine_insert;
wenzelm
parents: 18897
diff changeset
   293
      cases |> map_index (fn (i, ("", _)) => string_of_int (i + 1) | (_, (name, _)) => name);
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   294
    val elems = cases |> map (fn (_, (vars, _)) =>
19482
9f11af8f7ef9 tuned basic list operators (flat, maps, map_filter);
wenzelm
parents: 19300
diff changeset
   295
      Element.Constrains (vars |> map_filter (fn (x, SOME T) => SOME (x, T) | _ => NONE)));
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   296
    val concl = cases |> map (fn (_, (_, props)) => (("", []), map (rpair []) props));
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   297
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   298
    fun mk_stmt stmt ctxt =
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   299
      let
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   300
        val thesis =
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   301
          ObjectLogic.fixed_judgment (ProofContext.theory_of ctxt) AutoBind.thesisN;
18907
f984f22f1cb4 Proof.refine_insert;
wenzelm
parents: 18897
diff changeset
   302
        val atts = map Attrib.internal
f984f22f1cb4 Proof.refine_insert;
wenzelm
parents: 18897
diff changeset
   303
          [RuleCases.consumes (~ (length cases)), RuleCases.case_names names];
f984f22f1cb4 Proof.refine_insert;
wenzelm
parents: 18897
diff changeset
   304
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   305
        fun assume_case ((name, (vars, _)), (_, propp)) ctxt' =
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   306
          let
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   307
            val xs = map fst vars;
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   308
            val props = map fst propp;
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   309
            val (parms, ctxt'') =
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   310
              ctxt'
19897
fe661eb3b0e7 ProofContext: moved variable operations to struct Variable;
wenzelm
parents: 19844
diff changeset
   311
              |> fold Variable.declare_term props
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   312
              |> fold_map ProofContext.inferred_param xs;
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   313
            val asm = Term.list_all_free (parms, Logic.list_implies (props, thesis));
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   314
          in
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   315
            ctxt' |> (snd o ProofContext.add_fixes_i (map (fn x => (x, NONE, NoSyn)) xs));
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   316
            ctxt' |> ProofContext.add_assms_i ProofContext.assume_export
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   317
              [((name, [ContextRules.intro_query NONE]), [(asm, [])])]
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   318
            |>> (fn [(_, [th])] => th)
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   319
          end;
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   320
        val (ths, ctxt') = ctxt
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   321
          |> (snd o ProofContext.add_fixes_i [(AutoBind.thesisN, NONE, NoSyn)])
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   322
          |> fold_map assume_case (cases ~~ stmt)
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   323
          |-> (fn ths => ProofContext.note_thmss_i [((thatN, []), [(ths, [])])] #> #2 #> pair ths);
19585
70a1ce3b23ae removed 'concl is' patterns;
wenzelm
parents: 19482
diff changeset
   324
      in (([(("", atts), [(thesis, [])])], ths), ctxt') end;
18897
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   325
  in ((elems, concl), mk_stmt) end;
b31293969d4f obtain(_i): optional name for 'that';
wenzelm
parents: 18870
diff changeset
   326
17858
bc4db8cfd92f added 'guess', which derives the obtained context from the course of reasoning;
wenzelm
parents: 17357
diff changeset
   327
end;