src/Provers/classical.ML
changeset 7154 687657a3f7e6
parent 7132 5c31d06ead04
child 7230 4ca0d7839ff1
--- a/src/Provers/classical.ML	Mon Aug 02 17:58:46 1999 +0200
+++ b/src/Provers/classical.ML	Mon Aug 02 17:59:06 1999 +0200
@@ -172,6 +172,8 @@
   val xtra_intro_local: Proof.context attribute
   val delrule_local: Proof.context attribute
   val cla_modifiers: (Args.T list -> (Proof.context attribute * Args.T list)) list
+  val cla_meth: (claset -> tactic) -> Proof.context -> Proof.method
+  val cla_meth': (claset -> int -> tactic) -> Proof.context -> Proof.method
   val cla_method: (claset -> tactic) -> Args.src -> Proof.context -> Proof.method
   val cla_method': (claset -> int -> tactic) -> Args.src -> Proof.context -> Proof.method
   val single_tac: claset -> thm list -> int -> tactic