src/Pure/Isar/method.ML
changeset 25270 2ed7b34f58e6
parent 24116 9915c39e0820
child 25699 891fe6b71d3b
equal deleted inserted replaced
25269:f9090ae5cec9 25270:2ed7b34f58e6
    43   val assumption: Proof.context -> method
    43   val assumption: Proof.context -> method
    44   val close: bool -> Proof.context -> method
    44   val close: bool -> Proof.context -> method
    45   val trace: Proof.context -> thm list -> unit
    45   val trace: Proof.context -> thm list -> unit
    46   val rule_tac: thm list -> thm list -> int -> tactic
    46   val rule_tac: thm list -> thm list -> int -> tactic
    47   val some_rule_tac: thm list -> Proof.context -> thm list -> int -> tactic
    47   val some_rule_tac: thm list -> Proof.context -> thm list -> int -> tactic
       
    48   val intros_tac: thm list -> thm list -> tactic
    48   val rule: thm list -> method
    49   val rule: thm list -> method
    49   val erule: int -> thm list -> method
    50   val erule: int -> thm list -> method
    50   val drule: int -> thm list -> method
    51   val drule: int -> thm list -> method
    51   val frule: int -> thm list -> method
    52   val frule: int -> thm list -> method
    52   val iprover_tac: Proof.context -> int option -> int -> tactic
    53   val iprover_tac: Proof.context -> int option -> int -> tactic
   286 val frule = meth' (gen_arule_tac Tactic.forward_tac);
   287 val frule = meth' (gen_arule_tac Tactic.forward_tac);
   287 
   288 
   288 end;
   289 end;
   289 
   290 
   290 
   291 
       
   292 (* intros_tac -- pervasive search spanned by intro rules *)
       
   293 
       
   294 fun intros_tac intros facts =
       
   295   ALLGOALS (insert_tac facts THEN'
       
   296       REPEAT_ALL_NEW (resolve_tac intros))
       
   297     THEN Tactic.distinct_subgoals_tac;
       
   298 
       
   299 
   291 (* iprover -- intuitionistic proof search *)
   300 (* iprover -- intuitionistic proof search *)
   292 
   301 
   293 local
   302 local
   294 
   303 
   295 val remdups_tac = SUBGOAL (fn (g, i) =>
   304 val remdups_tac = SUBGOAL (fn (g, i) =>