removed internal functions from the signature (they are not needed anymore)
authorChristian Urban <urbanc@in.tum.de>
Thu, 13 May 2010 15:12:05 +0100
changeset 2123 2f39ce2aba6c
parent 2122 24ca435ead14
child 2124 a17b25cb94a6
removed internal functions from the signature (they are not needed anymore)
Nominal-General/nominal_thmdecls.ML
--- a/Nominal-General/nominal_thmdecls.ML	Thu May 13 10:34:59 2010 +0100
+++ b/Nominal-General/nominal_thmdecls.ML	Thu May 13 15:12:05 2010 +0100
@@ -35,10 +35,6 @@
   val get_eqvts_raw_thms: Proof.context -> thm list
   val eqvt_transform: Proof.context -> thm -> thm
   val is_eqvt: Proof.context -> term -> bool
-
-  (* TEMPORARY FIX *)
-  val add_thm: thm -> Context.generic -> Context.generic
-  val add_raw_thm: thm -> Context.generic -> Context.generic
 end;
 
 structure Nominal_ThmDecls: NOMINAL_THMDECLS =