src/Pure/goal.ML
author wenzelm
Mon, 06 Sep 2021 13:49:36 +0200
changeset 74248 ea9f2cb22e50
parent 74232 1091880266e5
child 74266 612b7e0d6721
permissions -rw-r--r--
more scalable operations;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/goal.ML
29345
5904873d8f11 tuned protect, conclude: Drule.comp_no_flatten;
wenzelm
parents: 29343
diff changeset
     2
    Author:     Makarius
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     3
49061
7449b804073b central management of forked goals wrt. transaction id;
wenzelm
parents: 49041
diff changeset
     4
Goals in tactical theorem proving, with support for forked proofs.
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     5
*)
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     6
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     7
signature BASIC_GOAL =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     8
sig
61527
d05f3d86a758 tuned signature -- clarified modules;
wenzelm
parents: 61508
diff changeset
     9
  val quick_and_dirty: bool Config.T
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    10
  val SELECT_GOAL: tactic -> int -> tactic
52458
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
    11
  val PREFER_GOAL: tactic -> int -> tactic
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
    12
  val CONJUNCTS: tactic -> int -> tactic
23414
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
    13
  val PRECISE_CONJUNCTS: int -> tactic -> int -> tactic
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    14
end;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    15
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    16
signature GOAL =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    17
sig
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    18
  include BASIC_GOAL
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    19
  val init: cterm -> thm
52456
960202346d0c tuned signature;
wenzelm
parents: 52223
diff changeset
    20
  val protect: int -> thm -> thm
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    21
  val conclude: thm -> thm
49845
9b19c0e81166 tuned signature;
wenzelm
parents: 49830
diff changeset
    22
  val check_finished: Proof.context -> thm -> thm
32197
bc341bbe4417 Goal.finish: explicit context for printing;
wenzelm
parents: 32187
diff changeset
    23
  val finish: Proof.context -> thm -> thm
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54742
diff changeset
    24
  val norm_result: Proof.context -> thm -> thm
52499
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
    25
  val skip_proofs_enabled: unit -> bool
28973
c549650d1442 future proofs: pass actual futures to facilitate composite computations;
wenzelm
parents: 28619
diff changeset
    26
  val future_result: Proof.context -> thm future -> term -> thm
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54742
diff changeset
    27
  val prove_internal: Proof.context -> cterm list -> cterm -> (thm list -> tactic) -> thm
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
    28
  val is_schematic: term -> bool
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
    29
  val prove_common: Proof.context -> int option -> string list -> term list -> term list ->
20290
3f886c176c9b normalized Proof.context/method type aliases;
wenzelm
parents: 20260
diff changeset
    30
    ({prems: thm list, context: Proof.context} -> tactic) -> thm list
28446
a01de3b3fa2e renamed promise to future, tuned related interfaces;
wenzelm
parents: 28363
diff changeset
    31
  val prove_future: Proof.context -> string list -> term list -> term ->
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
    32
    ({prems: thm list, context: Proof.context} -> tactic) -> thm
20290
3f886c176c9b normalized Proof.context/method type aliases;
wenzelm
parents: 20260
diff changeset
    33
  val prove: Proof.context -> string list -> term list -> term ->
3f886c176c9b normalized Proof.context/method type aliases;
wenzelm
parents: 20260
diff changeset
    34
    ({prems: thm list, context: Proof.context} -> tactic) -> thm
51118
32a5994dd205 tuned signature -- legacy packages might want to fork proofs as well;
wenzelm
parents: 51110
diff changeset
    35
  val prove_global_future: theory -> string list -> term list -> term ->
32a5994dd205 tuned signature -- legacy packages might want to fork proofs as well;
wenzelm
parents: 51110
diff changeset
    36
    ({prems: thm list, context: Proof.context} -> tactic) -> thm
26713
1c6181def1d0 prove_global: Variable.set_body true, pass context;
wenzelm
parents: 26628
diff changeset
    37
  val prove_global: theory -> string list -> term list -> term ->
1c6181def1d0 prove_global: Variable.set_body true, pass context;
wenzelm
parents: 26628
diff changeset
    38
    ({prems: thm list, context: Proof.context} -> tactic) -> thm
51551
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
    39
  val prove_sorry: Proof.context -> string list -> term list -> term ->
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
    40
    ({prems: thm list, context: Proof.context} -> tactic) -> thm
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
    41
  val prove_sorry_global: theory -> string list -> term list -> term ->
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
    42
    ({prems: thm list, context: Proof.context} -> tactic) -> thm
52458
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
    43
  val restrict: int -> int -> thm -> thm
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
    44
  val unrestrict: int -> thm -> thm
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
    45
  val conjunction_tac: int -> tactic
23414
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
    46
  val precise_conjunction_tac: int -> int -> tactic
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
    47
  val recover_conjunction_tac: tactic
54742
7a86358a3c0b proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
wenzelm
parents: 54567
diff changeset
    48
  val norm_hhf_tac: Proof.context -> int -> tactic
23237
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
    49
  val assume_rule_tac: Proof.context -> int -> tactic
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    50
end;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    51
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    52
structure Goal: GOAL =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    53
struct
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    54
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    55
(** goals **)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    56
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    57
(*
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    58
  -------- (init)
67721
5348bea4accd eliminated ASCII syntax from Pure bootstrap;
wenzelm
parents: 65458
diff changeset
    59
  C \<Longrightarrow> #C
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    60
*)
60642
48dd1cefb4ae simplified Thm.instantiate and derivatives: the LHS refers to non-certified variables -- this merely serves as index into already certified structures (or is ignored);
wenzelm
parents: 59623
diff changeset
    61
fun init C = Thm.instantiate ([], [((("A", 0), propT), C)]) Drule.protectI;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    62
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    63
(*
67721
5348bea4accd eliminated ASCII syntax from Pure bootstrap;
wenzelm
parents: 65458
diff changeset
    64
  A1 \<Longrightarrow> ... \<Longrightarrow> An \<Longrightarrow> C
52456
960202346d0c tuned signature;
wenzelm
parents: 52223
diff changeset
    65
  ------------------------ (protect n)
67721
5348bea4accd eliminated ASCII syntax from Pure bootstrap;
wenzelm
parents: 65458
diff changeset
    66
  A1 \<Longrightarrow> ... \<Longrightarrow> An \<Longrightarrow> #C
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    67
*)
52456
960202346d0c tuned signature;
wenzelm
parents: 52223
diff changeset
    68
fun protect n th = Drule.comp_no_flatten (th, n) 1 Drule.protectI;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    69
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    70
(*
67721
5348bea4accd eliminated ASCII syntax from Pure bootstrap;
wenzelm
parents: 65458
diff changeset
    71
  A \<Longrightarrow> ... \<Longrightarrow> #C
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    72
  ---------------- (conclude)
67721
5348bea4accd eliminated ASCII syntax from Pure bootstrap;
wenzelm
parents: 65458
diff changeset
    73
  A \<Longrightarrow> ... \<Longrightarrow> C
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    74
*)
29345
5904873d8f11 tuned protect, conclude: Drule.comp_no_flatten;
wenzelm
parents: 29343
diff changeset
    75
fun conclude th = Drule.comp_no_flatten (th, Thm.nprems_of th) 1 Drule.protectD;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    76
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    77
(*
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    78
  #C
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    79
  --- (finish)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    80
   C
17983
wenzelm
parents: 17980
diff changeset
    81
*)
32197
bc341bbe4417 Goal.finish: explicit context for printing;
wenzelm
parents: 32187
diff changeset
    82
fun check_finished ctxt th =
51608
wenzelm
parents: 51607
diff changeset
    83
  if Thm.no_prems th then th
wenzelm
parents: 51607
diff changeset
    84
  else
51958
bca32217b304 retain goal display options when printing error messages, to avoid breakdown for huge goals;
wenzelm
parents: 51608
diff changeset
    85
    raise THM ("Proof failed.\n" ^ Pretty.string_of (Goal_Display.pretty_goal ctxt th), 0, [th]);
32197
bc341bbe4417 Goal.finish: explicit context for printing;
wenzelm
parents: 32187
diff changeset
    86
49845
9b19c0e81166 tuned signature;
wenzelm
parents: 49830
diff changeset
    87
fun finish ctxt = check_finished ctxt #> conclude;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    88
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    89
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    90
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    91
(** results **)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    92
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
    93
(* normal form *)
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
    94
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54742
diff changeset
    95
fun norm_result ctxt =
58950
d07464875dd4 optional proof context for unify operations, for the sake of proper local options;
wenzelm
parents: 58837
diff changeset
    96
  Drule.flexflex_unique (SOME ctxt)
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54742
diff changeset
    97
  #> Raw_Simplifier.norm_hhf_protect ctxt
21604
1af327306c8e added norm/close_result (supercede local_standard etc.);
wenzelm
parents: 21579
diff changeset
    98
  #> Thm.strip_shyps
1af327306c8e added norm/close_result (supercede local_standard etc.);
wenzelm
parents: 21579
diff changeset
    99
  #> Drule.zero_var_indexes;
1af327306c8e added norm/close_result (supercede local_standard etc.);
wenzelm
parents: 21579
diff changeset
   100
1af327306c8e added norm/close_result (supercede local_standard etc.);
wenzelm
parents: 21579
diff changeset
   101
41703
d27950860514 parallelization of nested Isar proofs is subject to Goal.parallel_proofs_threshold;
wenzelm
parents: 41683
diff changeset
   102
(* scheduling parameters *)
d27950860514 parallelization of nested Isar proofs is subject to Goal.parallel_proofs_threshold;
wenzelm
parents: 41683
diff changeset
   103
52499
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   104
fun skip_proofs_enabled () =
52710
52790e3961fe just one option "skip_proofs", without direct access within the editor (it makes document processing stateful without strong reasons -- monotonic updates already handle goal forks smoothly);
wenzelm
parents: 52696
diff changeset
   105
  let val skip = Options.default_bool "skip_proofs" in
52499
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   106
    if Proofterm.proofs_enabled () andalso skip then
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   107
      (warning "Proof terms enabled -- cannot skip proofs"; false)
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   108
    else skip
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   109
  end;
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   110
29448
34b9652b2f45 added Goal.future_enabled abstraction -- now also checks that this is already
wenzelm
parents: 29435
diff changeset
   111
28446
a01de3b3fa2e renamed promise to future, tuned related interfaces;
wenzelm
parents: 28363
diff changeset
   112
(* future_result *)
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   113
28446
a01de3b3fa2e renamed promise to future, tuned related interfaces;
wenzelm
parents: 28363
diff changeset
   114
fun future_result ctxt result prop =
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   115
  let
30473
e0b66c11e7e4 Assumption.all_prems_of, Assumption.all_assms_of;
wenzelm
parents: 29448
diff changeset
   116
    val assms = Assumption.all_assms_of ctxt;
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   117
    val As = map Thm.term_of assms;
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   118
74248
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   119
    val frees = Term_Subst.Frees.build (fold Term_Subst.add_frees (prop :: As));
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   120
    val xs = Term_Subst.Frees.fold_rev (cons o Thm.cterm_of ctxt o Free o #1) frees [];
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   121
74248
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   122
    val tfrees = Term_Subst.TFrees.build (fold Term_Subst.add_tfrees (prop :: As));
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   123
    val Ts = Symtab.build (Term_Subst.TFrees.fold (Symtab.insert_set o #1 o #1) tfrees);
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   124
    val instT =
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   125
      build (tfrees |> Term_Subst.TFrees.fold (fn ((a, S), ()) =>
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   126
        cons (((a, 0), S), Thm.ctyp_of ctxt (TFree (a, S)))));
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   127
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   128
    val global_prop =
74248
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   129
      Logic.list_implies (As, prop)
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   130
      |> Term_Subst.Frees.fold_rev (Logic.all o Free o #1) frees
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   131
      |> Logic.varify_types_global
59623
920889b0788e clarified context;
wenzelm
parents: 59621
diff changeset
   132
      |> Thm.cterm_of ctxt
61508
2c7e2ae6173d clarified modules;
wenzelm
parents: 60948
diff changeset
   133
      |> Thm.weaken_sorts' ctxt;
28973
c549650d1442 future proofs: pass actual futures to facilitate composite computations;
wenzelm
parents: 28619
diff changeset
   134
    val global_result = result |> Future.map
58950
d07464875dd4 optional proof context for unify operations, for the sake of proper local options;
wenzelm
parents: 58837
diff changeset
   135
      (Drule.flexflex_unique (SOME ctxt) #>
28973
c549650d1442 future proofs: pass actual futures to facilitate composite computations;
wenzelm
parents: 28619
diff changeset
   136
        Drule.implies_intr_list assms #>
74248
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   137
        Drule.forall_intr_list xs #>
68693
a9bef20b1e47 proper adjust_maxidx: assms could have maxidx >= 0, e.g. from command "subgoal premises";
wenzelm
parents: 68130
diff changeset
   138
        Thm.adjust_maxidx_thm ~1 #>
74248
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   139
        Thm.generalize (Ts, Symtab.empty) 0 #>
70459
f0a445c5a82c maintain sort constraints from type instantiations, with pro-forma derivation to collect oracles/thms;
wenzelm
parents: 70398
diff changeset
   140
        Thm.strip_shyps #>
f0a445c5a82c maintain sort constraints from type instantiations, with pro-forma derivation to collect oracles/thms;
wenzelm
parents: 70398
diff changeset
   141
        Thm.solve_constraints);
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   142
    val local_result =
32056
f4b74cbecdaf future_result: explicitly impose Variable.sorts_of again;
wenzelm
parents: 30473
diff changeset
   143
      Thm.future global_result global_prop
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 70459
diff changeset
   144
      |> Thm.close_derivation \<^here>
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   145
      |> Thm.instantiate (instT, [])
74248
ea9f2cb22e50 more scalable operations;
wenzelm
parents: 74232
diff changeset
   146
      |> Drule.forall_elim_list xs
70459
f0a445c5a82c maintain sort constraints from type instantiations, with pro-forma derivation to collect oracles/thms;
wenzelm
parents: 70398
diff changeset
   147
      |> fold (Thm.elim_implies o Thm.assume) assms
f0a445c5a82c maintain sort constraints from type instantiations, with pro-forma derivation to collect oracles/thms;
wenzelm
parents: 70398
diff changeset
   148
      |> Thm.solve_constraints;
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   149
  in local_result end;
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   150
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   151
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   152
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   153
(** tactical theorem proving **)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   154
23356
dbe3731241c3 renamed prove_raw to prove_internal;
wenzelm
parents: 23237
diff changeset
   155
(* prove_internal -- minimal checks, no normalization of result! *)
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   156
54883
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54742
diff changeset
   157
fun prove_internal ctxt casms cprop tac =
dd04a8b654fc proper context for norm_hhf and derived operations;
wenzelm
parents: 54742
diff changeset
   158
  (case SINGLE (tac (map (Assumption.assume ctxt) casms)) (init cprop) of
54992
e5f4075d4c5e clarified context;
wenzelm
parents: 54985
diff changeset
   159
    SOME th => Drule.implies_intr_list casms (finish ctxt th)
38875
c7a66b584147 tuned messages: discontinued spurious full-stops (messages are occasionally composed unexpectedly);
wenzelm
parents: 38236
diff changeset
   160
  | NONE => error "Tactic failed");
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   161
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   162
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   163
(* prove variations *)
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   164
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   165
fun is_schematic t =
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   166
  Term.exists_subterm Term.is_Var t orelse
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   167
  Term.exists_type (Term.exists_subtype Term.is_TVar) t;
17986
0450847646c3 prove_raw: cterms, explicit asms;
wenzelm
parents: 17983
diff changeset
   168
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   169
fun prove_common ctxt fork_pri xs asms props tac =
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   170
  let
42360
da8817d01e7c modernized structure Proof_Context;
wenzelm
parents: 41819
diff changeset
   171
    val thy = Proof_Context.theory_of ctxt;
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   172
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   173
    val schematic = exists is_schematic props;
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   174
    val immediate = is_none fork_pri;
70398
725438ceae7c proof terms are always constructed sequentially;
wenzelm
parents: 69575
diff changeset
   175
    val future = Future.proofs_enabled 1 andalso not (Proofterm.proofs_enabled ());
52499
812215680f6d clarified Proofterm.proofs vs. Goal.skip_proofs;
wenzelm
parents: 52461
diff changeset
   176
    val skip = not immediate andalso not schematic andalso future andalso skip_proofs_enabled ();
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   177
28355
b9d9360e2440 prove: error with original thread position;
wenzelm
parents: 28341
diff changeset
   178
    val pos = Position.thread_data ();
55559
d4aea4bbe87f tuned message;
wenzelm
parents: 54994
diff changeset
   179
    fun err msg =
d4aea4bbe87f tuned message;
wenzelm
parents: 54994
diff changeset
   180
      cat_error msg
d4aea4bbe87f tuned message;
wenzelm
parents: 54994
diff changeset
   181
        ("The error(s) above occurred for the goal statement" ^ Position.here pos ^ ":\n" ^
d4aea4bbe87f tuned message;
wenzelm
parents: 54994
diff changeset
   182
          Syntax.string_of_term ctxt (Logic.list_implies (asms, Logic.mk_conjunction_list props)));
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   183
59623
920889b0788e clarified context;
wenzelm
parents: 59621
diff changeset
   184
    fun cert_safe t = Thm.cterm_of ctxt (Envir.beta_norm (Term.no_dummy_patterns t))
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   185
      handle TERM (msg, _) => err msg | TYPE (msg, _, _) => err msg;
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   186
    val casms = map cert_safe asms;
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   187
    val cprops = map cert_safe props;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   188
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   189
    val (prems, ctxt') = ctxt
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   190
      |> Variable.add_fixes_direct xs
27218
4548c83cd508 prove: full Variable.declare_term, including constraints;
wenzelm
parents: 26939
diff changeset
   191
      |> fold Variable.declare_term (asms @ props)
26713
1c6181def1d0 prove_global: Variable.set_body true, pass context;
wenzelm
parents: 26628
diff changeset
   192
      |> Assumption.add_assumes casms
1c6181def1d0 prove_global: Variable.set_body true, pass context;
wenzelm
parents: 26628
diff changeset
   193
      ||> Variable.set_body true;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   194
61508
2c7e2ae6173d clarified modules;
wenzelm
parents: 60948
diff changeset
   195
    val stmt = Thm.weaken_sorts' ctxt' (Conjunction.mk_conjunction_balanced cprops);
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   196
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   197
    fun tac' args st =
59498
50b60f501b05 proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents: 58963
diff changeset
   198
      if skip then ALLGOALS (Skip_Proof.cheat_tac ctxt) st before Skip_Proof.report ctxt
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   199
      else tac args st;
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   200
    fun result () =
51553
63327f679cff more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm
parents: 51552
diff changeset
   201
      (case SINGLE (tac' {prems = prems, context = ctxt'}) (init stmt) of
38875
c7a66b584147 tuned messages: discontinued spurious full-stops (messages are occasionally composed unexpectedly);
wenzelm
parents: 38236
diff changeset
   202
        NONE => err "Tactic failed"
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   203
      | SOME st =>
54567
cfe53047dc16 more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
wenzelm
parents: 53192
diff changeset
   204
          let
54981
a128df2f670e explicit check of background theory;
wenzelm
parents: 54883
diff changeset
   205
            val _ =
65458
cf504b7a7aa7 tuned signature;
wenzelm
parents: 64567
diff changeset
   206
              Context.subthy_id (Thm.theory_id st, Context.theory_id thy) orelse
59582
0fbed69ff081 tuned signature -- prefer qualified names;
wenzelm
parents: 59564
diff changeset
   207
                err "Bad background theory of goal state";
54567
cfe53047dc16 more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
wenzelm
parents: 53192
diff changeset
   208
            val res =
cfe53047dc16 more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
wenzelm
parents: 53192
diff changeset
   209
              (finish ctxt' st
58950
d07464875dd4 optional proof context for unify operations, for the sake of proper local options;
wenzelm
parents: 58837
diff changeset
   210
                |> Drule.flexflex_unique (SOME ctxt')
61508
2c7e2ae6173d clarified modules;
wenzelm
parents: 60948
diff changeset
   211
                |> Thm.check_shyps ctxt'
54994
8e98d67325b1 reactivate Thm.check_hyps, after adapting AFP/Datatype_Order_Generator (see AFP/b7e389b5765c);
wenzelm
parents: 54993
diff changeset
   212
                |> Thm.check_hyps (Context.Proof ctxt'))
54567
cfe53047dc16 more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
wenzelm
parents: 53192
diff changeset
   213
              handle THM (msg, _, _) => err msg | ERROR msg => err msg;
cfe53047dc16 more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
wenzelm
parents: 53192
diff changeset
   214
          in
58950
d07464875dd4 optional proof context for unify operations, for the sake of proper local options;
wenzelm
parents: 58837
diff changeset
   215
            if Unify.matches_list (Context.Proof ctxt') [Thm.term_of stmt] [Thm.prop_of res]
d07464875dd4 optional proof context for unify operations, for the sake of proper local options;
wenzelm
parents: 58837
diff changeset
   216
            then res
54567
cfe53047dc16 more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
wenzelm
parents: 53192
diff changeset
   217
            else err ("Proved a different theorem: " ^ Syntax.string_of_term ctxt' (Thm.prop_of res))
28340
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   218
          end);
e8597242f649 added promise_result, prove_promise;
wenzelm
parents: 27218
diff changeset
   219
    val res =
53192
04df1d236e1c maintain goal forks as part of global execution;
wenzelm
parents: 53190
diff changeset
   220
      if immediate orelse schematic orelse not future orelse skip then result ()
04df1d236e1c maintain goal forks as part of global execution;
wenzelm
parents: 53190
diff changeset
   221
      else
04df1d236e1c maintain goal forks as part of global execution;
wenzelm
parents: 53190
diff changeset
   222
        future_result ctxt'
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   223
          (Execution.fork {name = "Goal.prove", pos = Position.thread_data (), pri = the fork_pri}
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   224
            result)
53192
04df1d236e1c maintain goal forks as part of global execution;
wenzelm
parents: 53190
diff changeset
   225
          (Thm.term_of stmt);
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   226
  in
60722
a8babbb6d5ea normalize proof before splitting conjunctions, according to Proof.conclude_goal (see also 4dd0ba632e40) -- may reduce general resource usage;
wenzelm
parents: 60695
diff changeset
   227
    res
70494
41108e3e9ca5 formal position for PThm nodes;
wenzelm
parents: 70459
diff changeset
   228
    |> Thm.close_derivation \<^here>
60722
a8babbb6d5ea normalize proof before splitting conjunctions, according to Proof.conclude_goal (see also 4dd0ba632e40) -- may reduce general resource usage;
wenzelm
parents: 60695
diff changeset
   229
    |> Conjunction.elim_balanced (length props)
20290
3f886c176c9b normalized Proof.context/method type aliases;
wenzelm
parents: 20260
diff changeset
   230
    |> map (Assumption.export false ctxt' ctxt)
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   231
    |> Variable.export ctxt' ctxt
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   232
    |> map Drule.zero_var_indexes
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   233
  end;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   234
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   235
fun prove_future_pri ctxt pri xs asms prop tac =
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   236
  hd (prove_common ctxt (SOME pri) xs asms [prop] tac);
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   237
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   238
fun prove_future ctxt = prove_future_pri ctxt ~1;
51118
32a5994dd205 tuned signature -- legacy packages might want to fork proofs as well;
wenzelm
parents: 51110
diff changeset
   239
59564
fdc03c8daacc Goal.prove_multi is superseded by the fully general Goal.prove_common;
wenzelm
parents: 59498
diff changeset
   240
fun prove ctxt xs asms prop tac = hd (prove_common ctxt NONE xs asms [prop] tac);
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   241
51118
32a5994dd205 tuned signature -- legacy packages might want to fork proofs as well;
wenzelm
parents: 51110
diff changeset
   242
fun prove_global_future thy xs asms prop tac =
32a5994dd205 tuned signature -- legacy packages might want to fork proofs as well;
wenzelm
parents: 51110
diff changeset
   243
  Drule.export_without_context (prove_future (Proof_Context.init_global thy) xs asms prop tac);
32a5994dd205 tuned signature -- legacy packages might want to fork proofs as well;
wenzelm
parents: 51110
diff changeset
   244
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   245
fun prove_global thy xs asms prop tac =
42360
da8817d01e7c modernized structure Proof_Context;
wenzelm
parents: 41819
diff changeset
   246
  Drule.export_without_context (prove (Proof_Context.init_global thy) xs asms prop tac);
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   247
61527
d05f3d86a758 tuned signature -- clarified modules;
wenzelm
parents: 61508
diff changeset
   248
d05f3d86a758 tuned signature -- clarified modules;
wenzelm
parents: 61508
diff changeset
   249
(* skip proofs *)
d05f3d86a758 tuned signature -- clarified modules;
wenzelm
parents: 61508
diff changeset
   250
69575
f77cc54f6d47 clarified signature: more types;
wenzelm
parents: 68693
diff changeset
   251
val quick_and_dirty = Config.declare_option_bool ("quick_and_dirty", \<^here>);
61527
d05f3d86a758 tuned signature -- clarified modules;
wenzelm
parents: 61508
diff changeset
   252
51551
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
   253
fun prove_sorry ctxt xs asms prop tac =
52059
2f970c7f722b proper option quick_and_dirty;
wenzelm
parents: 51958
diff changeset
   254
  if Config.get ctxt quick_and_dirty then
59498
50b60f501b05 proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents: 58963
diff changeset
   255
    prove ctxt xs asms prop (fn _ => ALLGOALS (Skip_Proof.cheat_tac ctxt))
68130
6fb85346cb79 clarified future scheduling parameters, with support for parallel_limit;
wenzelm
parents: 68025
diff changeset
   256
  else (if Future.proofs_enabled 1 then prove_future_pri ctxt ~2 else prove ctxt) xs asms prop tac;
51551
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
   257
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
   258
fun prove_sorry_global thy xs asms prop tac =
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
   259
  Drule.export_without_context
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
   260
    (prove_sorry (Proof_Context.init_global thy) xs asms prop tac);
88d1d19fb74f tuned signature and module arrangement;
wenzelm
parents: 51423
diff changeset
   261
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   262
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   263
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   264
(** goal structure **)
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   265
52458
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   266
(* rearrange subgoals *)
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   267
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   268
fun restrict i n st =
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   269
  if i < 1 orelse n < 1 orelse i + n - 1 > Thm.nprems_of st
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   270
  then raise THM ("Goal.restrict", i, [st])
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   271
  else rotate_prems (i - 1) st |> protect n;
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   272
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   273
fun unrestrict i = conclude #> rotate_prems (1 - i);
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   274
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   275
(*with structural marker*)
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   276
fun SELECT_GOAL tac i st =
19191
56cda3ec2ef8 SELECT_GOAL: fixed trivial case;
wenzelm
parents: 19184
diff changeset
   277
  if Thm.nprems_of st = 1 andalso i = 1 then tac st
52458
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   278
  else (PRIMITIVE (restrict i 1) THEN tac THEN PRIMITIVE (unrestrict i)) st;
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   279
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   280
(*without structural marker*)
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   281
fun PREFER_GOAL tac i st =
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   282
  if i < 1 orelse i > Thm.nprems_of st then Seq.empty
210bca64b894 less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
wenzelm
parents: 52456
diff changeset
   283
  else (PRIMITIVE (rotate_prems (i - 1)) THEN tac THEN PRIMITIVE (rotate_prems (1 - i))) st;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   284
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   285
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   286
(* multiple goals *)
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   287
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   288
fun precise_conjunction_tac 0 i = eq_assume_tac i
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   289
  | precise_conjunction_tac 1 i = SUBGOAL (K all_tac) i
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   290
  | precise_conjunction_tac n i = PRIMITIVE (Drule.with_subgoal i (Conjunction.curry_balanced n));
23414
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
   291
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   292
val adhoc_conjunction_tac = REPEAT_ALL_NEW
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   293
  (SUBGOAL (fn (goal, i) =>
59498
50b60f501b05 proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents: 58963
diff changeset
   294
    if can Logic.dest_conjunction goal then resolve0_tac [Conjunction.conjunctionI] i
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   295
    else no_tac));
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   296
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   297
val conjunction_tac = SUBGOAL (fn (goal, i) =>
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   298
  precise_conjunction_tac (length (Logic.dest_conjunctions goal)) i ORELSE
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   299
  TRY (adhoc_conjunction_tac i));
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   300
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   301
val recover_conjunction_tac = PRIMITIVE (fn th =>
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   302
  Conjunction.uncurry_balanced (Thm.nprems_of th) th);
23414
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
   303
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
   304
fun PRECISE_CONJUNCTS n tac =
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
   305
  SELECT_GOAL (precise_conjunction_tac n 1
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
   306
    THEN tac
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   307
    THEN recover_conjunction_tac);
23414
927203ad4b3a tuned conjunction tactics: slightly smaller proof terms;
wenzelm
parents: 23356
diff changeset
   308
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   309
fun CONJUNCTS tac =
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   310
  SELECT_GOAL (conjunction_tac 1
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   311
    THEN tac
23418
c195f6f13769 balanced conjunctions;
wenzelm
parents: 23414
diff changeset
   312
    THEN recover_conjunction_tac);
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   313
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   314
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   315
(* hhf normal form *)
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   316
54742
7a86358a3c0b proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
wenzelm
parents: 54567
diff changeset
   317
fun norm_hhf_tac ctxt =
59498
50b60f501b05 proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents: 58963
diff changeset
   318
  resolve_tac ctxt [Drule.asm_rl]  (*cheap approximation -- thanks to builtin Logic.flatten_params*)
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   319
  THEN' SUBGOAL (fn (t, i) =>
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   320
    if Drule.is_norm_hhf t then all_tac
54742
7a86358a3c0b proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
wenzelm
parents: 54567
diff changeset
   321
    else rewrite_goal_tac ctxt Drule.norm_hhf_eqs i);
21687
f689f729afab reorganized structure Goal vs. Tactic;
wenzelm
parents: 21604
diff changeset
   322
23237
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   323
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   324
(* non-atomic goal assumptions *)
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   325
56245
84fc7dfa3cd4 more qualified names;
wenzelm
parents: 55559
diff changeset
   326
fun non_atomic (Const ("Pure.imp", _) $ _ $ _) = true
84fc7dfa3cd4 more qualified names;
wenzelm
parents: 55559
diff changeset
   327
  | non_atomic (Const ("Pure.all", _) $ _) = true
23356
dbe3731241c3 renamed prove_raw to prove_internal;
wenzelm
parents: 23237
diff changeset
   328
  | non_atomic _ = false;
dbe3731241c3 renamed prove_raw to prove_internal;
wenzelm
parents: 23237
diff changeset
   329
54742
7a86358a3c0b proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
wenzelm
parents: 54567
diff changeset
   330
fun assume_rule_tac ctxt = norm_hhf_tac ctxt THEN' CSUBGOAL (fn (goal, i) =>
23237
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   331
  let
60695
757549b4bbe6 Variable.focus etc.: optional bindings provided by user;
wenzelm
parents: 60642
diff changeset
   332
    val ((_, goal'), ctxt') = Variable.focus_cterm NONE goal ctxt;
23237
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   333
    val goal'' = Drule.cterm_rule (singleton (Variable.export ctxt' ctxt)) goal';
23356
dbe3731241c3 renamed prove_raw to prove_internal;
wenzelm
parents: 23237
diff changeset
   334
    val Rs = filter (non_atomic o Thm.term_of) (Drule.strip_imp_prems goal'');
23237
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   335
    val tacs = Rs |> map (fn R =>
59498
50b60f501b05 proper context for resolve_tac, eresolve_tac, dresolve_tac, forward_tac etc.;
wenzelm
parents: 58963
diff changeset
   336
      eresolve_tac ctxt [Raw_Simplifier.norm_hhf ctxt (Thm.trivial R)] THEN_ALL_NEW assume_tac ctxt);
23237
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   337
  in fold_rev (curry op APPEND') tacs (K no_tac) i end);
ac9d126456e1 added assume_rule_tac;
wenzelm
parents: 22902
diff changeset
   338
52461
ef4c16887f83 more scalable PARALLEL_GOALS, using more elementary retrofit;
wenzelm
parents: 52458
diff changeset
   339
end;
ef4c16887f83 more scalable PARALLEL_GOALS, using more elementary retrofit;
wenzelm
parents: 52458
diff changeset
   340
32365
9b74d0339c44 added PARALLEL_CHOICE, PARALLEL_GOALS;
wenzelm
parents: 32255
diff changeset
   341
structure Basic_Goal: BASIC_GOAL = Goal;
9b74d0339c44 added PARALLEL_CHOICE, PARALLEL_GOALS;
wenzelm
parents: 32255
diff changeset
   342
open Basic_Goal;