do not export standard_infer_types;
authorwenzelm
Fri, 19 Oct 2007 16:13:53 +0200
changeset 25097 796190c7918d
parent 25096 b8950f7cf92e
child 25098 1ec53c9ae71a
do not export standard_infer_types;
src/Pure/Isar/proof_context.ML
--- a/src/Pure/Isar/proof_context.ML	Fri Oct 19 15:08:33 2007 +0200
+++ b/src/Pure/Isar/proof_context.ML	Fri Oct 19 16:13:53 2007 +0200
@@ -144,7 +144,6 @@
   val add_const_constraint: string * typ option -> Proof.context -> Proof.context
   val add_abbrev: string -> Markup.property list ->
     bstring * term -> Proof.context -> (term * term) * Proof.context
-  val standard_infer_types: Proof.context -> term list -> term list
   val revert_abbrev: string -> string -> Proof.context -> Proof.context
   val verbose: bool ref
   val setmp_verbose: ('a -> 'b) -> 'a -> 'b