src/Pure/Isar/overloading.ML
changeset 38377 2dfd8b7b8274
parent 38342 09d4a04d5c2e
child 38381 7d1e2a6831ec
--- a/src/Pure/Isar/overloading.ML	Wed Aug 11 15:09:30 2010 +0200
+++ b/src/Pure/Isar/overloading.ML	Wed Aug 11 15:09:31 2010 +0200
@@ -6,14 +6,6 @@
 
 signature OVERLOADING =
 sig
-  val init: (string * (string * typ) * bool) list -> theory -> Proof.context
-  val conclude: local_theory -> local_theory
-  val declare: string * typ -> theory -> term * theory
-  val confirm: binding -> local_theory -> local_theory
-  val define: bool -> binding -> string * term -> theory -> thm * theory
-  val operation: Proof.context -> binding -> (string * bool) option
-  val pretty: Proof.context -> Pretty.T
-
   type improvable_syntax
   val add_improvable_syntax: Proof.context -> Proof.context
   val map_improvable_syntax: (improvable_syntax -> improvable_syntax)