src/Pure/goal.ML
author wenzelm
Sun, 30 Jul 2006 21:28:52 +0200
changeset 20260 990dbc007ca6
parent 20250 c3f209752749
child 20290 3f886c176c9b
permissions -rw-r--r--
Thm.adjust_maxidx;
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     1
(*  Title:      Pure/goal.ML
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     2
    ID:         $Id$
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     3
    Author:     Makarius and Lawrence C Paulson
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     4
18139
wenzelm
parents: 18119
diff changeset
     5
Goals in tactical theorem proving.
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     6
*)
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     7
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     8
signature BASIC_GOAL =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
     9
sig
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    10
  val SELECT_GOAL: tactic -> int -> tactic
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    11
end;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    12
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    13
signature GOAL =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    14
sig
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    15
  include BASIC_GOAL
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    16
  val init: cterm -> thm
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    17
  val protect: thm -> thm
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    18
  val conclude: thm -> thm
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    19
  val finish: thm -> thm
18119
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    20
  val compose_hhf: thm -> int -> thm -> thm Seq.seq
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    21
  val compose_hhf_tac: thm -> int -> tactic
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    22
  val comp_hhf: thm -> thm -> thm
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    23
  val prove_raw: cterm list -> cterm -> (thm list -> tactic) -> thm
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
    24
  val prove_multi: Context.proof -> string list -> term list -> term list ->
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    25
    ({prems: thm list, context: Context.proof} -> tactic) -> thm list
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    26
  val prove: Context.proof -> string list -> term list -> term ->
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    27
    ({prems: thm list, context: Context.proof} -> tactic) -> thm
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
    28
  val prove_global: theory -> string list -> term list -> term -> (thm list -> tactic) -> thm
19184
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
    29
  val extract: int -> int -> thm -> thm Seq.seq
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
    30
  val retrofit: int -> int -> thm -> thm -> thm Seq.seq
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    31
end;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    32
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    33
structure Goal: GOAL =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    34
struct
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    35
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    36
(** goals **)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    37
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    38
(*
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    39
  -------- (init)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    40
  C ==> #C
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    41
*)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    42
fun init ct = Drule.instantiate' [] [SOME ct] Drule.protectI;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    43
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    44
(*
18119
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    45
   C
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    46
  --- (protect)
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    47
  #C
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    48
*)
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    49
fun protect th = th COMP Drule.incr_indexes th Drule.protectI;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    50
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    51
(*
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    52
  A ==> ... ==> #C
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    53
  ---------------- (conclude)
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    54
  A ==> ... ==> C
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    55
*)
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    56
fun conclude th =
18497
7569674d7bb1 Thm.compose_no_flatten;
wenzelm
parents: 18484
diff changeset
    57
  (case SINGLE (Thm.compose_no_flatten false (th, Thm.nprems_of th) 1)
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    58
      (Drule.incr_indexes th Drule.protectD) of
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    59
    SOME th' => th'
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    60
  | NONE => raise THM ("Failed to conclude goal", 0, [th]));
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    61
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    62
(*
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    63
  #C
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    64
  --- (finish)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    65
   C
17983
wenzelm
parents: 17980
diff changeset
    66
*)
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    67
fun finish th =
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    68
  (case Thm.nprems_of th of
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    69
    0 => conclude th
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    70
  | n => raise THM ("Proof failed.\n" ^
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    71
      Pretty.string_of (Pretty.chunks (Display.pretty_goals n th)) ^
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    72
      ("\n" ^ string_of_int n ^ " unsolved goal(s)!"), 0, [th]));
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    73
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
    74
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    75
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    76
(** results **)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    77
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    78
(* composition of normal results *)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    79
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    80
fun compose_hhf tha i thb =
18145
6757627acf59 renamed Thm.cgoal_of to Thm.cprem_of;
wenzelm
parents: 18139
diff changeset
    81
  Thm.bicompose false (false, Drule.lift_all (Thm.cprem_of thb i) tha, 0) i thb;
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    82
18119
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    83
fun compose_hhf_tac th i = PRIMSEQ (compose_hhf th i);
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    84
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    85
fun comp_hhf tha thb =
19862
7f29aa958b72 Unify.matches_list;
wenzelm
parents: 19774
diff changeset
    86
  (case Seq.chop 2 (compose_hhf tha 1 thb) of
18119
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    87
    ([th], _) => th
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    88
  | ([], _) => raise THM ("comp_hhf: no unifiers", 1, [tha, thb])
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
    89
  | _  => raise THM ("comp_hhf: multiple unifiers", 1, [tha, thb]));
17986
0450847646c3 prove_raw: cterms, explicit asms;
wenzelm
parents: 17983
diff changeset
    90
0450847646c3 prove_raw: cterms, explicit asms;
wenzelm
parents: 17983
diff changeset
    91
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    92
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    93
(** tactical theorem proving **)
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
    94
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    95
(* prove_raw -- no checks, no normalization of result! *)
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    96
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    97
fun prove_raw casms cprop tac =
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    98
  (case SINGLE (tac (map Assumption.assume casms)) (init cprop) of
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
    99
    SOME th => Drule.implies_intr_list casms (finish th)
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   100
  | NONE => error "Tactic failed.");
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   101
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   102
18119
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
   103
(* prove_multi *)
17986
0450847646c3 prove_raw: cterms, explicit asms;
wenzelm
parents: 17983
diff changeset
   104
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   105
fun prove_multi ctxt xs asms props tac =
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   106
  let
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   107
    val thy = Context.theory_of_proof ctxt;
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   108
    val string_of_term = Sign.string_of_term thy;
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   109
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   110
    fun err msg = cat_error msg
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   111
      ("The error(s) above occurred for the goal statement:\n" ^
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   112
        string_of_term (Logic.list_implies (asms, Logic.mk_conjunction_list props)));
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   113
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   114
    fun cert_safe t = Thm.cterm_of thy (Envir.beta_norm (Term.no_dummy_patterns t))
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   115
      handle TERM (msg, _) => err msg | TYPE (msg, _, _) => err msg;
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   116
    val casms = map cert_safe asms;
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   117
    val cprops = map cert_safe props;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   118
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   119
    val (prems, ctxt') = ctxt
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   120
      |> Variable.add_fixes_direct xs
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   121
      |> fold Variable.declare_internal (asms @ props)
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   122
      |> Assumption.add_assumes casms;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   123
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   124
    val goal = init (Conjunction.mk_conjunction_list cprops);
19774
5fe7731d0836 allow non-trivial schematic goals (via embedded term vars);
wenzelm
parents: 19619
diff changeset
   125
    val res =
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   126
      (case SINGLE (tac {prems = prems, context = ctxt'}) goal of
19774
5fe7731d0836 allow non-trivial schematic goals (via embedded term vars);
wenzelm
parents: 19619
diff changeset
   127
        NONE => err "Tactic failed."
5fe7731d0836 allow non-trivial schematic goals (via embedded term vars);
wenzelm
parents: 19619
diff changeset
   128
      | SOME res => res);
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   129
    val [results] = Conjunction.elim_precise [length props] (finish res)
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   130
      handle THM (msg, _, _) => err msg;
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   131
    val _ = Unify.matches_list thy (map Thm.term_of cprops) (map Thm.prop_of results)
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   132
      orelse err ("Proved a different theorem: " ^ string_of_term (Thm.prop_of res));
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   133
  in
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   134
    results
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   135
    |> (Seq.hd o Assumption.exports false ctxt' ctxt)
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   136
    |> Variable.export ctxt' ctxt
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   137
    |> map Drule.zero_var_indexes
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   138
  end;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   139
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   140
18119
63901a9b99dc export compose_hhf;
wenzelm
parents: 18027
diff changeset
   141
(* prove *)
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   142
20056
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   143
fun prove ctxt xs asms prop tac = hd (prove_multi ctxt xs asms [prop] tac);
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   144
0698a403a066 prove/prove_multi: context;
wenzelm
parents: 19862
diff changeset
   145
fun prove_global thy xs asms prop tac =
20250
c3f209752749 prove: proper assumption context, more tactic arguments;
wenzelm
parents: 20228
diff changeset
   146
  Drule.standard (prove (Context.init_proof thy) xs asms prop (fn {prems, ...} => tac prems));
18027
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   147
09ab79d4e8e1 renamed Goal constant to prop, more general protect/unprotect interfaces;
wenzelm
parents: 17986
diff changeset
   148
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   149
19184
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
   150
(** local goal states **)
18207
9edbeda7e39a tuned norm_hhf_protected;
wenzelm
parents: 18180
diff changeset
   151
19184
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
   152
fun extract i n st =
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
   153
  (if i < 1 orelse n < 1 orelse i + n - 1 > Thm.nprems_of st then Seq.empty
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
   154
   else if n = 1 then Seq.single (Thm.cprem_of st i)
19423
51eeee99bd8f use conjunction stuff from conjunction.ML;
wenzelm
parents: 19221
diff changeset
   155
   else Seq.single (foldr1 Conjunction.mk_conjunction (map (Thm.cprem_of st) (i upto i + n - 1))))
20260
990dbc007ca6 Thm.adjust_maxidx;
wenzelm
parents: 20250
diff changeset
   156
  |> Seq.map (Thm.adjust_maxidx_cterm ~1 #> init);
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   157
19221
wenzelm
parents: 19191
diff changeset
   158
fun retrofit i n st' st =
wenzelm
parents: 19191
diff changeset
   159
  (if n = 1 then st
19423
51eeee99bd8f use conjunction stuff from conjunction.ML;
wenzelm
parents: 19221
diff changeset
   160
   else st |> Drule.rotate_prems (i - 1) |> Conjunction.uncurry n |> Drule.rotate_prems (1 - i))
19221
wenzelm
parents: 19191
diff changeset
   161
  |> Thm.compose_no_flatten false (conclude st', Thm.nprems_of st') i;
18207
9edbeda7e39a tuned norm_hhf_protected;
wenzelm
parents: 18180
diff changeset
   162
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   163
fun SELECT_GOAL tac i st =
19191
56cda3ec2ef8 SELECT_GOAL: fixed trivial case;
wenzelm
parents: 19184
diff changeset
   164
  if Thm.nprems_of st = 1 andalso i = 1 then tac st
19184
3e30297e1300 added extract, retrofit;
wenzelm
parents: 18678
diff changeset
   165
  else Seq.lifts (retrofit i 1) (Seq.maps tac (extract i 1 st)) st;
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   166
18207
9edbeda7e39a tuned norm_hhf_protected;
wenzelm
parents: 18180
diff changeset
   167
end;
9edbeda7e39a tuned norm_hhf_protected;
wenzelm
parents: 18180
diff changeset
   168
17980
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   169
structure BasicGoal: BASIC_GOAL = Goal;
788836292b1a Internal goals.
wenzelm
parents:
diff changeset
   170
open BasicGoal;