src/Provers/classical.ML
changeset 61327 0a4c364df431
parent 61268 abe08fb15a12
child 61853 fb7756087101
--- a/src/Provers/classical.ML	Mon Oct 05 14:17:20 2015 +0200
+++ b/src/Provers/classical.ML	Mon Oct 05 18:03:52 2015 +0200
@@ -119,6 +119,8 @@
   val unsafe_elim: int option -> attribute
   val unsafe_intro: int option -> attribute
   val rule_del: attribute
+  val rule_tac: Proof.context -> thm list -> thm list -> int -> tactic
+  val standard_tac: Proof.context -> thm list -> tactic
   val cla_modifiers: Method.modifier parser list
   val cla_method:
     (Proof.context -> tactic) -> (Proof.context -> Proof.method) context_parser