export proof method in signature
authorblanchet
Thu, 01 Oct 2015 17:35:28 +0200
changeset 61302 9f9b088d8824
parent 61301 484f7878ede4
child 61303 af6b8bd0d076
export proof method in signature
src/HOL/Tools/Metis/metis_tactic.ML
--- a/src/HOL/Tools/Metis/metis_tactic.ML	Thu Oct 01 17:32:07 2015 +0200
+++ b/src/HOL/Tools/Metis/metis_tactic.ML	Thu Oct 01 17:35:28 2015 +0200
@@ -16,6 +16,8 @@
   val metis_tac_unused : string list -> string -> Proof.context -> thm list -> int -> thm ->
     thm list * thm Seq.seq
   val metis_tac : string list -> string -> Proof.context -> thm list -> int -> tactic
+  val metis_method : (string list option * string option) * thm list -> Proof.context -> thm list ->
+    thm -> thm Seq.seq
   val metis_lam_transs : string list
   val parse_metis_options : (string list option * string option) parser
 end