added function store_termination_rule to the signature, as it is used in Nominal2
authorChristian Urban <urbanc@in.tum.de>
Sun, 28 Oct 2012 02:22:39 +0000
changeset 49979 4de92b4aa74a
parent 49978 c163145dd40f
child 49980 34b0464d7eef
added function store_termination_rule to the signature, as it is used in Nominal2
src/HOL/Tools/Function/function_common.ML
--- a/src/HOL/Tools/Function/function_common.ML	Sat Oct 27 20:59:50 2012 +0200
+++ b/src/HOL/Tools/Function/function_common.ML	Sun Oct 28 02:22:39 2012 +0000
@@ -72,6 +72,7 @@
   structure Termination_Simps: NAMED_THMS
   val set_termination_prover : (Proof.context -> tactic) -> Context.generic -> Context.generic
   val get_termination_prover : Proof.context -> tactic
+  val store_termination_rule : thm -> Context.generic -> Context.generic
   datatype function_config = FunctionConfig of
    {sequential: bool,
     default: string option,