src/Pure/tactic.ML
changeset 214 ed6a3e2b1a33
parent 191 fe5d88d4c7e1
child 230 ec8a2b6aa8a7
equal deleted inserted replaced
213:42f2b8a3581f 214:ed6a3e2b1a33
    11   structure Tactical: TACTICAL and Net: NET
    11   structure Tactical: TACTICAL and Net: NET
    12   local open Tactical Tactical.Thm Net
    12   local open Tactical Tactical.Thm Net
    13   in
    13   in
    14   val ares_tac: thm list -> int -> tactic
    14   val ares_tac: thm list -> int -> tactic
    15   val asm_rewrite_goal_tac:
    15   val asm_rewrite_goal_tac:
    16         (meta_simpset -> tactic) -> meta_simpset -> int -> tactic
    16         bool*bool -> (meta_simpset -> tactic) -> meta_simpset -> int -> tactic
    17   val assume_tac: int -> tactic
    17   val assume_tac: int -> tactic
    18   val atac: int ->tactic
    18   val atac: int ->tactic
    19   val bimatch_from_nets_tac: (int*(bool*thm)) net * (int*(bool*thm)) net -> int -> tactic
    19   val bimatch_from_nets_tac: (int*(bool*thm)) net * (int*(bool*thm)) net -> int -> tactic
    20   val bimatch_tac: (bool*thm)list -> int -> tactic
    20   val bimatch_tac: (bool*thm)list -> int -> tactic
    21   val biresolve_from_nets_tac: (int*(bool*thm)) net * (int*(bool*thm)) net -> int -> tactic
    21   val biresolve_from_nets_tac: (int*(bool*thm)) net * (int*(bool*thm)) net -> int -> tactic
   371   case Sequence.pull(tapply(tacf mss,thm)) of
   371   case Sequence.pull(tapply(tacf mss,thm)) of
   372     None => None
   372     None => None
   373   | Some(thm,_) => Some(thm);
   373   | Some(thm,_) => Some(thm);
   374 
   374 
   375 (*Rewrite subgoal i only *)
   375 (*Rewrite subgoal i only *)
   376 fun asm_rewrite_goal_tac prover_tac mss i =
   376 fun asm_rewrite_goal_tac mode prover_tac mss i =
   377       PRIMITIVE(rewrite_goal_rule (result1 prover_tac) mss i);
   377       PRIMITIVE(rewrite_goal_rule mode (result1 prover_tac) mss i);
   378 
   378 
   379 (*Rewrite throughout proof state. *)
   379 (*Rewrite throughout proof state. *)
   380 fun rewrite_tac defs = PRIMITIVE(rewrite_rule defs);
   380 fun rewrite_tac defs = PRIMITIVE(rewrite_rule defs);
   381 
   381 
   382 (*Rewrite subgoals only, not main goal. *)
   382 (*Rewrite subgoals only, not main goal. *)