| author | paulson | 
| Wed, 28 Jun 2000 10:56:01 +0200 | |
| changeset 9172 | 2dbb80d4fdb7 | 
| parent 8535 | 7428194b39f7 | 
| child 10767 | 8fa4aafa7314 | 
| permissions | -rw-r--r-- | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 1 | (* Title: tctical | 
| 0 | 2 | ID: $Id$ | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 3 | Author: Lawrence C Paulson, Cambridge University Computer Laboratory | 
| 0 | 4 | Copyright 1993 University of Cambridge | 
| 5 | ||
| 6 | Tacticals | |
| 7 | *) | |
| 8 | ||
| 4602 | 9 | infix 1 THEN THEN' THEN_ALL_NEW; | 
| 0 | 10 | infix 0 ORELSE APPEND INTLEAVE ORELSE' APPEND' INTLEAVE'; | 
| 671 | 11 | infix 0 THEN_ELSE; | 
| 12 | ||
| 0 | 13 | |
| 14 | signature TACTICAL = | |
| 15 | sig | |
| 4270 | 16 | type tactic (* = thm -> thm Seq.seq*) | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 17 | val all_tac : tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 18 | val ALLGOALS : (int -> tactic) -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 19 | val APPEND : tactic * tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 20 |   val APPEND'           : ('a -> tactic) * ('a -> tactic) -> 'a -> tactic
 | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 21 | val CHANGED : tactic -> tactic | 
| 5141 | 22 | val CHANGED_GOAL : (int -> tactic) -> int -> tactic | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 23 | val COND : (thm -> bool) -> tactic -> tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 24 | val DETERM : tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 25 | val EVERY : tactic list -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 26 |   val EVERY'            : ('a -> tactic) list -> 'a -> tactic
 | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 27 | val EVERY1 : (int -> tactic) list -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 28 | val FILTER : (thm -> bool) -> tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 29 | val FIRST : tactic list -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 30 |   val FIRST'            : ('a -> tactic) list -> 'a -> tactic
 | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 31 | val FIRST1 : (int -> tactic) list -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 32 | val FIRSTGOAL : (int -> tactic) -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 33 | val goals_limit : int ref | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 34 | val INTLEAVE : tactic * tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 35 |   val INTLEAVE'         : ('a -> tactic) * ('a -> tactic) -> 'a -> tactic
 | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 36 | val METAHYPS : (thm list -> tactic) -> int -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 37 | val no_tac : tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 38 | val ORELSE : tactic * tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 39 |   val ORELSE'           : ('a -> tactic) * ('a -> tactic) -> 'a -> tactic
 | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 40 | val pause_tac : tactic | 
| 6041 | 41 | val print_tac : string -> tactic | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 42 | val REPEAT : tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 43 | val REPEAT1 : tactic -> tactic | 
| 8149 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 44 | val REPEAT_FIRST : (int -> tactic) -> tactic | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 45 | val REPEAT_SOME : (int -> tactic) -> tactic | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 46 | val REPEAT_DETERM_N : int -> tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 47 | val REPEAT_DETERM : tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 48 | val REPEAT_DETERM1 : tactic -> tactic | 
| 703 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 49 | val REPEAT_DETERM_FIRST: (int -> tactic) -> tactic | 
| 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 50 | val REPEAT_DETERM_SOME: (int -> tactic) -> tactic | 
| 8149 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 51 | val DETERM_UNTIL : (thm -> bool) -> tactic -> tactic | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 52 | val SELECT_GOAL : tactic -> int -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 53 | val SOMEGOAL : (int -> tactic) -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 54 | val strip_context : term -> (string * typ) list * term list * term | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 55 | val SUBGOAL : ((term*int) -> tactic) -> int -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 56 | val suppress_tracing : bool ref | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 57 | val THEN : tactic * tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 58 |   val THEN'             : ('a -> tactic) * ('a -> tactic) -> 'a -> tactic
 | 
| 4602 | 59 | val THEN_ALL_NEW : (int -> tactic) * (int -> tactic) -> int -> tactic | 
| 8341 | 60 | val REPEAT_ALL_NEW : (int -> tactic) -> int -> tactic | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 61 | val THEN_ELSE : tactic * (tactic*tactic) -> tactic | 
| 4270 | 62 | val traced_tac : (thm -> (thm * thm Seq.seq) option) -> tactic | 
| 5141 | 63 | val tracify : bool ref -> tactic -> tactic | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 64 | val trace_REPEAT : bool ref | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 65 | val TRY : tactic -> tactic | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 66 | val TRYALL : (int -> tactic) -> tactic | 
| 0 | 67 | end; | 
| 68 | ||
| 69 | ||
| 1502 | 70 | structure Tactical : TACTICAL = | 
| 0 | 71 | struct | 
| 72 | ||
| 73 | (**** Tactics ****) | |
| 74 | ||
| 75 | (*A tactic maps a proof tree to a sequence of proof trees: | |
| 76 | if length of sequence = 0 then the tactic does not apply; | |
| 77 | if length > 1 then backtracking on the alternatives can occur.*) | |
| 78 | ||
| 4270 | 79 | type tactic = thm -> thm Seq.seq; | 
| 0 | 80 | |
| 81 | ||
| 82 | (*** LCF-style tacticals ***) | |
| 83 | ||
| 84 | (*the tactical THEN performs one tactic followed by another*) | |
| 4270 | 85 | fun (tac1 THEN tac2) st = Seq.flat (Seq.map tac2 (tac1 st)); | 
| 0 | 86 | |
| 87 | ||
| 88 | (*The tactical ORELSE uses the first tactic that returns a nonempty sequence. | |
| 89 | Like in LCF, ORELSE commits to either tac1 or tac2 immediately. | |
| 90 | Does not backtrack to tac2 if tac1 was initially chosen. *) | |
| 1502 | 91 | fun (tac1 ORELSE tac2) st = | 
| 4270 | 92 | case Seq.pull(tac1 st) of | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 93 | None => tac2 st | 
| 4270 | 94 | | sequencecell => Seq.make(fn()=> sequencecell); | 
| 0 | 95 | |
| 96 | ||
| 97 | (*The tactical APPEND combines the results of two tactics. | |
| 98 | Like ORELSE, but allows backtracking on both tac1 and tac2. | |
| 99 | The tactic tac2 is not applied until needed.*) | |
| 1502 | 100 | fun (tac1 APPEND tac2) st = | 
| 4270 | 101 | Seq.append(tac1 st, | 
| 102 | Seq.make(fn()=> Seq.pull (tac2 st))); | |
| 0 | 103 | |
| 104 | (*Like APPEND, but interleaves results of tac1 and tac2.*) | |
| 1502 | 105 | fun (tac1 INTLEAVE tac2) st = | 
| 4270 | 106 | Seq.interleave(tac1 st, | 
| 107 | Seq.make(fn()=> Seq.pull (tac2 st))); | |
| 0 | 108 | |
| 671 | 109 | (*Conditional tactic. | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 110 | tac1 ORELSE tac2 = tac1 THEN_ELSE (all_tac, tac2) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 111 | tac1 THEN tac2 = tac1 THEN_ELSE (tac2, no_tac) | 
| 671 | 112 | *) | 
| 1502 | 113 | fun (tac THEN_ELSE (tac1, tac2)) st = | 
| 4270 | 114 | case Seq.pull(tac st) of | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 115 | None => tac2 st (*failed; try tactic 2*) | 
| 4270 | 116 | | seqcell => Seq.flat (*succeeded; use tactic 1*) | 
| 117 | (Seq.map tac1 (Seq.make(fn()=> seqcell))); | |
| 671 | 118 | |
| 119 | ||
| 0 | 120 | (*Versions for combining tactic-valued functions, as in | 
| 121 | SOMEGOAL (resolve_tac rls THEN' assume_tac) *) | |
| 1502 | 122 | fun (tac1 THEN' tac2) x = tac1 x THEN tac2 x; | 
| 123 | fun (tac1 ORELSE' tac2) x = tac1 x ORELSE tac2 x; | |
| 124 | fun (tac1 APPEND' tac2) x = tac1 x APPEND tac2 x; | |
| 125 | fun (tac1 INTLEAVE' tac2) x = tac1 x INTLEAVE tac2 x; | |
| 0 | 126 | |
| 127 | (*passes all proofs through unchanged; identity of THEN*) | |
| 4270 | 128 | fun all_tac st = Seq.single st; | 
| 0 | 129 | |
| 130 | (*passes no proofs through; identity of ORELSE and APPEND*) | |
| 4270 | 131 | fun no_tac st = Seq.empty; | 
| 0 | 132 | |
| 133 | ||
| 134 | (*Make a tactic deterministic by chopping the tail of the proof sequence*) | |
| 1502 | 135 | fun DETERM tac st = | 
| 4270 | 136 | case Seq.pull (tac st) of | 
| 137 | None => Seq.empty | |
| 138 | | Some(x,_) => Seq.cons(x, Seq.empty); | |
| 0 | 139 | |
| 140 | ||
| 141 | (*Conditional tactical: testfun controls which tactic to use next. | |
| 142 | Beware: due to eager evaluation, both thentac and elsetac are evaluated.*) | |
| 1502 | 143 | fun COND testfun thenf elsef = (fn prf => | 
| 0 | 144 | if testfun prf then thenf prf else elsef prf); | 
| 145 | ||
| 146 | (*Do the tactic or else do nothing*) | |
| 147 | fun TRY tac = tac ORELSE all_tac; | |
| 148 | ||
| 2672 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 149 | (*** List-oriented tactics ***) | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 150 | |
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 151 | local | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 152 | (*This version of EVERY avoids backtracking over repeated states*) | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 153 | |
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 154 | fun EVY (trail, []) st = | 
| 4270 | 155 | Seq.make (fn()=> Some(st, | 
| 156 | Seq.make (fn()=> Seq.pull (evyBack trail)))) | |
| 2672 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 157 | | EVY (trail, tac::tacs) st = | 
| 4270 | 158 | case Seq.pull(tac st) of | 
| 2672 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 159 | None => evyBack trail (*failed: backtrack*) | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 160 | | Some(st',q) => EVY ((st',q,tacs)::trail, tacs) st' | 
| 4270 | 161 | and evyBack [] = Seq.empty (*no alternatives*) | 
| 2672 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 162 | | evyBack ((st',q,tacs)::trail) = | 
| 4270 | 163 | case Seq.pull q of | 
| 2672 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 164 | None => evyBack trail | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 165 | | Some(st,q') => if eq_thm (st',st) | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 166 | then evyBack ((st',q',tacs)::trail) | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 167 | else EVY ((st,q',tacs)::trail, tacs) st | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 168 | in | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 169 | |
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 170 | (* EVERY [tac1,...,tacn] equals tac1 THEN ... THEN tacn *) | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 171 | fun EVERY tacs = EVY ([], tacs); | 
| 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 172 | end; | 
| 2627 | 173 | |
| 0 | 174 | |
| 1502 | 175 | (* EVERY' [tac1,...,tacn] i equals tac1 i THEN ... THEN tacn i *) | 
| 2672 
85d7e800d754
Replaced "flat" by the Basis Library function List.concat
 paulson parents: 
2627diff
changeset | 176 | fun EVERY' tacs i = EVERY (map (fn f => f i) tacs); | 
| 0 | 177 | |
| 178 | (*Apply every tactic to 1*) | |
| 1502 | 179 | fun EVERY1 tacs = EVERY' tacs 1; | 
| 0 | 180 | |
| 181 | (* FIRST [tac1,...,tacn] equals tac1 ORELSE ... ORELSE tacn *) | |
| 182 | fun FIRST tacs = foldr (op ORELSE) (tacs, no_tac); | |
| 183 | ||
| 1502 | 184 | (* FIRST' [tac1,...,tacn] i equals tac1 i ORELSE ... ORELSE tacn i *) | 
| 185 | fun FIRST' tacs = foldr (op ORELSE') (tacs, K no_tac); | |
| 0 | 186 | |
| 187 | (*Apply first tactic to 1*) | |
| 1502 | 188 | fun FIRST1 tacs = FIRST' tacs 1; | 
| 0 | 189 | |
| 190 | ||
| 191 | (*** Tracing tactics ***) | |
| 192 | ||
| 193 | (*Max number of goals to print -- set by user*) | |
| 194 | val goals_limit = ref 10; | |
| 195 | ||
| 196 | (*Print the current proof state and pass it on.*) | |
| 6041 | 197 | fun print_tac msg = | 
| 1502 | 198 | (fn st => | 
| 6041 | 199 | (writeln msg; | 
| 200 | print_goals (!goals_limit) st; Seq.single st)); | |
| 0 | 201 | |
| 202 | (*Pause until a line is typed -- if non-empty then fail. *) | |
| 1502 | 203 | fun pause_tac st = | 
| 5957 | 204 | (writeln "** Press RETURN to continue:"; | 
| 4270 | 205 | if TextIO.inputLine TextIO.stdIn = "\n" then Seq.single st | 
| 5956 | 206 | else (writeln "Goodbye"; Seq.empty)); | 
| 0 | 207 | |
| 208 | exception TRACE_EXIT of thm | |
| 209 | and TRACE_QUIT; | |
| 210 | ||
| 631 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 211 | (*Tracing flags*) | 
| 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 212 | val trace_REPEAT= ref false | 
| 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 213 | and suppress_tracing = ref false; | 
| 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 214 | |
| 0 | 215 | (*Handle all tracing commands for current state and tactic *) | 
| 1502 | 216 | fun exec_trace_command flag (tac, st) = | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 217 | case TextIO.inputLine(TextIO.stdIn) of | 
| 1502 | 218 | "\n" => tac st | 
| 4270 | 219 | | "f\n" => Seq.empty | 
| 1502 | 220 | | "o\n" => (flag:=false; tac st) | 
| 221 | | "s\n" => (suppress_tracing:=true; tac st) | |
| 5956 | 222 | | "x\n" => (writeln "Exiting now"; raise (TRACE_EXIT st)) | 
| 0 | 223 | | "quit\n" => raise TRACE_QUIT | 
| 5956 | 224 | | _ => (writeln | 
| 0 | 225 | "Type RETURN to continue or...\n\ | 
| 226 | \ f - to fail here\n\ | |
| 227 | \ o - to switch tracing off\n\ | |
| 631 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 228 | \ s - to suppress tracing until next entry to a tactical\n\ | 
| 0 | 229 | \ x - to exit at this point\n\ | 
| 230 | \ quit - to abort this tracing run\n\ | |
| 1502 | 231 | \** Well? " ; exec_trace_command flag (tac, st)); | 
| 0 | 232 | |
| 233 | ||
| 234 | (*Extract from a tactic, a thm->thm seq function that handles tracing*) | |
| 1502 | 235 | fun tracify flag tac st = | 
| 631 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 236 | if !flag andalso not (!suppress_tracing) | 
| 3669 
3384c6f1f095
removed print_goals_ref (which was broken anyway);
 wenzelm parents: 
3561diff
changeset | 237 | then (print_goals (!goals_limit) st; | 
| 5957 | 238 | writeln "** Press RETURN to continue:"; | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 239 | exec_trace_command flag (tac,st)) | 
| 1502 | 240 | else tac st; | 
| 0 | 241 | |
| 242 | (*Create a tactic whose outcome is given by seqf, handling TRACE_EXIT*) | |
| 1502 | 243 | fun traced_tac seqf st = | 
| 631 
8bc44f7bbab8
Pure/tctical/suppress_tracing: new; can now switch tracing off until the
 lcp parents: 
230diff
changeset | 244 | (suppress_tracing := false; | 
| 4270 | 245 | Seq.make (fn()=> seqf st | 
| 246 | handle TRACE_EXIT st' => Some(st', Seq.empty))); | |
| 0 | 247 | |
| 248 | ||
| 8149 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 249 | (*Deterministic DO..UNTIL: only retains the first outcome; tail recursive. | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 250 | Forces repitition until predicate on state is fulfilled.*) | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 251 | fun DETERM_UNTIL p tac = | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 252 | let val tac = tracify trace_REPEAT tac | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 253 | fun drep st = if p st then Some (st, Seq.empty) | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 254 | else (case Seq.pull(tac st) of | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 255 | None => None | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 256 | | Some(st',_) => drep st') | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 257 | in traced_tac drep end; | 
| 
941afb897532
added tacticals DETERM_UNTIL and DETERM_UNTIL_SOLVED
 oheimb parents: 
7686diff
changeset | 258 | |
| 0 | 259 | (*Deterministic REPEAT: only retains the first outcome; | 
| 703 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 260 | uses less space than REPEAT; tail recursive. | 
| 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 261 | If non-negative, n bounds the number of repetitions.*) | 
| 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 262 | fun REPEAT_DETERM_N n tac = | 
| 1502 | 263 | let val tac = tracify trace_REPEAT tac | 
| 4270 | 264 | fun drep 0 st = Some(st, Seq.empty) | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 265 | | drep n st = | 
| 4270 | 266 | (case Seq.pull(tac st) of | 
| 267 | None => Some(st, Seq.empty) | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 268 | | Some(st',_) => drep (n-1) st') | 
| 703 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 269 | in traced_tac (drep n) end; | 
| 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 270 | |
| 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 271 | (*Allows any number of repetitions*) | 
| 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 272 | val REPEAT_DETERM = REPEAT_DETERM_N ~1; | 
| 0 | 273 | |
| 274 | (*General REPEAT: maintains a stack of alternatives; tail recursive*) | |
| 275 | fun REPEAT tac = | |
| 1502 | 276 | let val tac = tracify trace_REPEAT tac | 
| 0 | 277 | fun rep qs st = | 
| 4270 | 278 | case Seq.pull(tac st) of | 
| 279 | None => Some(st, Seq.make(fn()=> repq qs)) | |
| 0 | 280 | | Some(st',q) => rep (q::qs) st' | 
| 281 | and repq [] = None | |
| 4270 | 282 | | repq(q::qs) = case Seq.pull q of | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 283 | None => repq qs | 
| 0 | 284 | | Some(st,q) => rep (q::qs) st | 
| 285 | in traced_tac (rep []) end; | |
| 286 | ||
| 287 | (*Repeat 1 or more times*) | |
| 703 
3a5cd2883581
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
 lcp parents: 
671diff
changeset | 288 | fun REPEAT_DETERM1 tac = DETERM tac THEN REPEAT_DETERM tac; | 
| 0 | 289 | fun REPEAT1 tac = tac THEN REPEAT tac; | 
| 290 | ||
| 291 | ||
| 292 | (** Filtering tacticals **) | |
| 293 | ||
| 294 | (*Returns all states satisfying the predicate*) | |
| 4270 | 295 | fun FILTER pred tac st = Seq.filter pred (tac st); | 
| 0 | 296 | |
| 297 | (*Returns all changed states*) | |
| 1643 
3f83b629f2e3
Fixed error in CHANGED (caused by variable renaming)
 paulson parents: 
1583diff
changeset | 298 | fun CHANGED tac st = | 
| 
3f83b629f2e3
Fixed error in CHANGED (caused by variable renaming)
 paulson parents: 
1583diff
changeset | 299 | let fun diff st' = not (eq_thm(st,st')) | 
| 4270 | 300 | in Seq.filter diff (tac st) end; | 
| 0 | 301 | |
| 302 | ||
| 303 | (*** Tacticals based on subgoal numbering ***) | |
| 304 | ||
| 1502 | 305 | (*For n subgoals, performs tac(n) THEN ... THEN tac(1) | 
| 306 | Essential to work backwards since tac(i) may add/delete subgoals at i. *) | |
| 307 | fun ALLGOALS tac st = | |
| 308 | let fun doall 0 = all_tac | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 309 | | doall n = tac(n) THEN doall(n-1) | 
| 1502 | 310 | in doall(nprems_of st)st end; | 
| 0 | 311 | |
| 1502 | 312 | (*For n subgoals, performs tac(n) ORELSE ... ORELSE tac(1) *) | 
| 313 | fun SOMEGOAL tac st = | |
| 314 | let fun find 0 = no_tac | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 315 | | find n = tac(n) ORELSE find(n-1) | 
| 1502 | 316 | in find(nprems_of st)st end; | 
| 0 | 317 | |
| 1502 | 318 | (*For n subgoals, performs tac(1) ORELSE ... ORELSE tac(n). | 
| 0 | 319 | More appropriate than SOMEGOAL in some cases.*) | 
| 1502 | 320 | fun FIRSTGOAL tac st = | 
| 321 | let fun find (i,n) = if i>n then no_tac else tac(i) ORELSE find (i+1,n) | |
| 322 | in find(1, nprems_of st)st end; | |
| 0 | 323 | |
| 1502 | 324 | (*Repeatedly solve some using tac. *) | 
| 325 | fun REPEAT_SOME tac = REPEAT1 (SOMEGOAL (REPEAT1 o tac)); | |
| 326 | fun REPEAT_DETERM_SOME tac = REPEAT_DETERM1 (SOMEGOAL (REPEAT_DETERM1 o tac)); | |
| 0 | 327 | |
| 1502 | 328 | (*Repeatedly solve the first possible subgoal using tac. *) | 
| 329 | fun REPEAT_FIRST tac = REPEAT1 (FIRSTGOAL (REPEAT1 o tac)); | |
| 330 | fun REPEAT_DETERM_FIRST tac = REPEAT_DETERM1 (FIRSTGOAL (REPEAT_DETERM1 o tac)); | |
| 0 | 331 | |
| 1502 | 332 | (*For n subgoals, tries to apply tac to n,...1 *) | 
| 333 | fun TRYALL tac = ALLGOALS (TRY o tac); | |
| 0 | 334 | |
| 335 | ||
| 336 | (*Make a tactic for subgoal i, if there is one. *) | |
| 2580 
e3f680709487
Gradual switching to Basis Library functions nth, drop, etc.
 paulson parents: 
2244diff
changeset | 337 | fun SUBGOAL goalfun i st = goalfun (List.nth(prems_of st, i-1), i) st | 
| 4270 | 338 | handle Subscript => Seq.empty; | 
| 0 | 339 | |
| 5141 | 340 | (*Returns all states that have changed in subgoal i, counted from the LAST | 
| 341 | subgoal. For stac, for example.*) | |
| 342 | fun CHANGED_GOAL tac i st = | |
| 7686 | 343 | let val np = nprems_of st | 
| 344 | val d = np-i (*distance from END*) | |
| 5141 | 345 | val t = List.nth(prems_of st, i-1) | 
| 7686 | 346 | fun diff st' = | 
| 347 | nprems_of st' - d <= 0 (*the subgoal no longer exists*) | |
| 348 | orelse | |
| 349 | not (Pattern.aeconv (t, | |
| 350 | List.nth(prems_of st', | |
| 351 | nprems_of st' - d - 1))) | |
| 5141 | 352 | in Seq.filter diff (tac i st) end | 
| 353 | handle Subscript => Seq.empty (*no subgoal i*); | |
| 354 | ||
| 4602 | 355 | fun (tac1 THEN_ALL_NEW tac2) i st = | 
| 8535 | 356 | st |> (tac1 i THEN (fn st' => Seq.INTERVAL tac2 i (i + nprems_of st' - nprems_of st) st')); | 
| 4602 | 357 | |
| 8341 | 358 | (*repeatedly dig into any emerging subgoals*) | 
| 359 | fun REPEAT_ALL_NEW tac = | |
| 360 | tac THEN_ALL_NEW (TRY o (fn i => REPEAT_ALL_NEW tac i)); | |
| 361 | ||
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 362 | |
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 363 | (*** SELECT_GOAL ***) | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 364 | |
| 0 | 365 | (*Tactical for restricting the effect of a tactic to subgoal i. | 
| 1502 | 366 | Works by making a new state from subgoal i, applying tac to it, and | 
| 0 | 367 | composing the resulting metathm with the original state. | 
| 368 | The "main goal" of the new state will not be atomic, some tactics may fail! | |
| 369 | DOES NOT work if tactic affects the main goal other than by instantiation.*) | |
| 370 | ||
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 371 | (*SELECT_GOAL optimization: replace the conclusion by a variable X, | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 372 | to avoid copying. Proof states have X==concl as an assuption.*) | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 373 | |
| 6390 | 374 | val prop_equals = cterm_of (Theory.sign_of ProtoPure.thy) | 
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 375 |                     (Const("==", propT-->propT-->propT));
 | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 376 | |
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 377 | fun mk_prop_equals(t,u) = capply (capply prop_equals t) u; | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 378 | |
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 379 | (*Like trivial but returns [ct==X] ct==>X instead of ct==>ct, if possible. | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 380 | It is paired with a function to undo the transformation. If ct contains | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 381 | Vars then it returns ct==>ct.*) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 382 | |
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 383 | fun eq_trivial ct = | 
| 6390 | 384 | let val xfree = cterm_of (Theory.sign_of ProtoPure.thy) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 385 | (Free (gensym"EQ_TRIVIAL_", propT)) | 
| 2158 
77dfe65b5bb3
Renamed SELECT_GOAL's new parameter from x to selct to avoid clashes
 paulson parents: 
2005diff
changeset | 386 | val ct_eq_x = mk_prop_equals (ct, xfree) | 
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 387 | and refl_ct = reflexive ct | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 388 | fun restore th = | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 389 | implies_elim | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 390 | (forall_elim ct (forall_intr xfree (implies_intr ct_eq_x th))) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 391 | refl_ct | 
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 392 | in (equal_elim | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 393 | (combination (combination refl_implies refl_ct) (assume ct_eq_x)) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 394 | (Drule.mk_triv_goal ct), | 
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 395 | restore) | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 396 | end (*Fails if there are Vars or TVars*) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 397 | handle THM _ => (Drule.mk_triv_goal ct, I); | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 398 | |
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 399 | |
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 400 | (*Does the work of SELECT_GOAL. *) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 401 | fun select tac st i = | 
| 2580 
e3f680709487
Gradual switching to Basis Library functions nth, drop, etc.
 paulson parents: 
2244diff
changeset | 402 | let val (eq_cprem, restore) = (*we hope maxidx goes to ~1*) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 403 | eq_trivial (adjust_maxidx (List.nth(cprems_of st, i-1))) | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 404 | fun next st' = | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 405 | let val np' = nprems_of st' | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 406 | (*rename the ?A in rev_triv_goal*) | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 407 | 	      val {maxidx,...} = rep_thm st'
 | 
| 6390 | 408 | val ct = cterm_of (Theory.sign_of ProtoPure.thy) | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 409 | 		                (Var(("A",maxidx+1), propT))
 | 
| 5906 | 410 | val rev_triv_goal' = instantiate' [] [Some ct] Drule.rev_triv_goal | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 411 | fun bic th = bicompose false (false, th, np') | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 412 | in bic (Seq.hd (bic (restore st') 1 rev_triv_goal')) i st end | 
| 4270 | 413 | in Seq.flat (Seq.map next (tac eq_cprem)) | 
| 2005 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 414 | end; | 
| 
a52f53caf424
Optimized version of SELECT_GOAL, up to 10% faster
 paulson parents: 
1643diff
changeset | 415 | |
| 1502 | 416 | fun SELECT_GOAL tac i st = | 
| 5312 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 417 | let val np = nprems_of st | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 418 | in if 1<=i andalso i<=np then | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 419 | (*If only one subgoal, then just apply tactic*) | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 420 | if np=1 then tac st else select tac st i | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 421 | else Seq.empty | 
| 
b380921982b9
simpler SELECT_GOAL no longer inserts a dummy parameter
 paulson parents: 
5141diff
changeset | 422 | end; | 
| 0 | 423 | |
| 424 | ||
| 425 | (*Strips assumptions in goal yielding ( [x1,...,xm], [H1,...,Hn], B ) | |
| 426 | H1,...,Hn are the hypotheses; x1...xm are variants of the parameters. | |
| 427 | Main difference from strip_assums concerns parameters: | |
| 428 | it replaces the bound variables by free variables. *) | |
| 429 | fun strip_context_aux (params, Hs, Const("==>", _) $ H $ B) = 
 | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 430 | strip_context_aux (params, H::Hs, B) | 
| 0 | 431 |   | strip_context_aux (params, Hs, Const("all",_)$Abs(a,T,t)) =
 | 
| 432 | let val (b,u) = variant_abs(a,T,t) | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 433 | in strip_context_aux ((b,T)::params, Hs, u) end | 
| 0 | 434 | | strip_context_aux (params, Hs, B) = (rev params, rev Hs, B); | 
| 435 | ||
| 436 | fun strip_context A = strip_context_aux ([],[],A); | |
| 437 | ||
| 438 | ||
| 439 | (**** METAHYPS -- tactical for using hypotheses as meta-level assumptions | |
| 1502 | 440 | METAHYPS (fn prems => tac prems) i | 
| 0 | 441 | |
| 442 | converts subgoal i, of the form !!x1...xm. [| A1;...;An] ==> A into a new | |
| 443 | proof state A==>A, supplying A1,...,An as meta-level assumptions (in | |
| 444 | "prems"). The parameters x1,...,xm become free variables. If the | |
| 445 | resulting proof state is [| B1;...;Bk] ==> C (possibly assuming A1,...,An) | |
| 446 | then it is lifted back into the original context, yielding k subgoals. | |
| 447 | ||
| 448 | Replaces unknowns in the context by Frees having the prefix METAHYP_ | |
| 449 | New unknowns in [| B1;...;Bk] ==> C are lifted over x1,...,xm. | |
| 450 | DOES NOT HANDLE TYPE UNKNOWNS. | |
| 451 | ****) | |
| 452 | ||
| 453 | local | |
| 454 | ||
| 455 | (*Left-to-right replacements: ctpairs = [...,(vi,ti),...]. | |
| 456 | Instantiates distinct free variables by terms of same type.*) | |
| 457 | fun free_instantiate ctpairs = | |
| 458 | forall_elim_list (map snd ctpairs) o forall_intr_list (map fst ctpairs); | |
| 459 | ||
| 460 | fun free_of s ((a,i), T) = | |
| 461 | Free(s ^ (case i of 0 => a | _ => a ^ "_" ^ string_of_int i), | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 462 | T) | 
| 0 | 463 | |
| 464 | fun mk_inst (var as Var(v,T)) = (var, free_of "METAHYP1_" (v,T)) | |
| 465 | in | |
| 466 | ||
| 1502 | 467 | fun metahyps_aux_tac tacf (prem,i) state = | 
| 0 | 468 |   let val {sign,maxidx,...} = rep_thm state
 | 
| 230 | 469 | val cterm = cterm_of sign | 
| 0 | 470 | (*find all vars in the hyps -- should find tvars also!*) | 
| 1502 | 471 | val hyps_vars = foldr add_term_vars (Logic.strip_assums_hyp prem, []) | 
| 0 | 472 | val insts = map mk_inst hyps_vars | 
| 473 | (*replace the hyps_vars by Frees*) | |
| 474 | val prem' = subst_atomic insts prem | |
| 475 | val (params,hyps,concl) = strip_context prem' | |
| 476 | val fparams = map Free params | |
| 477 | val cparams = map cterm fparams | |
| 478 | and chyps = map cterm hyps | |
| 479 | val hypths = map assume chyps | |
| 480 | fun swap_ctpair (t,u) = (cterm u, cterm t) | |
| 481 | (*Subgoal variables: make Free; lift type over params*) | |
| 482 | fun mk_subgoal_inst concl_vars (var as Var(v,T)) = | |
| 483 | if var mem concl_vars | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 484 | then (var, true, free_of "METAHYP2_" (v,T)) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 485 | else (var, false, | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 486 | free_of "METAHYP2_" (v, map #2 params --->T)) | 
| 0 | 487 | (*Instantiate subgoal vars by Free applied to params*) | 
| 488 | fun mk_ctpair (t,in_concl,u) = | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 489 | if in_concl then (cterm t, cterm u) | 
| 0 | 490 | else (cterm t, cterm (list_comb (u,fparams))) | 
| 491 | (*Restore Vars with higher type and index*) | |
| 492 | fun mk_subgoal_swap_ctpair | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 493 | (t as Var((a,i),_), in_concl, u as Free(_,U)) = | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 494 | if in_concl then (cterm u, cterm t) | 
| 0 | 495 | else (cterm u, cterm(Var((a, i+maxidx), U))) | 
| 496 | (*Embed B in the original context of params and hyps*) | |
| 1502 | 497 | fun embed B = list_all_free (params, Logic.list_implies (hyps, B)) | 
| 0 | 498 | (*Strip the context using elimination rules*) | 
| 499 | fun elim Bhyp = implies_elim_list (forall_elim_list cparams Bhyp) hypths | |
| 500 | (*Embed an ff pair in the original params*) | |
| 1502 | 501 | fun embed_ff(t,u) = Logic.mk_flexpair (list_abs_free (params, t), | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 502 | list_abs_free (params, u)) | 
| 0 | 503 | (*Remove parameter abstractions from the ff pairs*) | 
| 504 | fun elim_ff ff = flexpair_abs_elim_list cparams ff | |
| 505 | (*A form of lifting that discharges assumptions.*) | |
| 506 | fun relift st = | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 507 | let val prop = #prop(rep_thm st) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 508 | val subgoal_vars = (*Vars introduced in the subgoals*) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 509 | foldr add_term_vars (Logic.strip_imp_prems prop, []) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 510 | and concl_vars = add_term_vars (Logic.strip_imp_concl prop, []) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 511 | val subgoal_insts = map (mk_subgoal_inst concl_vars) subgoal_vars | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 512 | val st' = instantiate ([], map mk_ctpair subgoal_insts) st | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 513 | val emBs = map (cterm o embed) (prems_of st') | 
| 0 | 514 | and ffs = map (cterm o embed_ff) (tpairs_of st') | 
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 515 | val Cth = implies_elim_list st' | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 516 | (map (elim_ff o assume) ffs @ | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 517 | map (elim o assume) emBs) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 518 | in (*restore the unknowns to the hypotheses*) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 519 | free_instantiate (map swap_ctpair insts @ | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 520 | map mk_subgoal_swap_ctpair subgoal_insts) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 521 | (*discharge assumptions from state in same order*) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 522 | (implies_intr_list (ffs@emBs) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 523 | (forall_intr_list cparams (implies_intr_list chyps Cth))) | 
| 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 524 | end | 
| 0 | 525 | val subprems = map (forall_elim_vars 0) hypths | 
| 526 | and st0 = trivial (cterm concl) | |
| 527 | (*function to replace the current subgoal*) | |
| 528 | fun next st = bicompose false (false, relift st, nprems_of st) | |
| 2244 
dacee519738a
Converted I/O operatios for Basis Library compatibility
 paulson parents: 
2158diff
changeset | 529 | i state | 
| 4270 | 530 | in Seq.flat (Seq.map next (tacf subprems st0)) | 
| 1502 | 531 | end; | 
| 0 | 532 | end; | 
| 533 | ||
| 534 | fun METAHYPS tacf = SUBGOAL (metahyps_aux_tac tacf); | |
| 535 | ||
| 536 | end; | |
| 1502 | 537 | |
| 538 | open Tactical; |