src/HOL/Tools/Quotient/quotient_info.ML
changeset 45278 7c6c8e950636
parent 45274 252cd58847e0
child 45279 89a17197cb98
--- a/src/HOL/Tools/Quotient/quotient_info.ML	Thu Oct 27 16:28:34 2011 +0200
+++ b/src/HOL/Tools/Quotient/quotient_info.ML	Thu Oct 27 19:41:08 2011 +0200
@@ -10,7 +10,6 @@
 sig
 
   type maps_info = {mapfun: string, relmap: string}
-  val maps_defined: theory -> string -> bool
   val maps_lookup: theory -> string -> maps_info option
   val maps_update_thy: string -> maps_info -> theory -> theory
   val maps_update: string -> maps_info -> Proof.context -> Proof.context
@@ -62,8 +61,6 @@
   fun merge data = Symtab.merge (K true) data
 )
 
-fun maps_defined thy s = Symtab.defined (MapsData.get thy) s
-
 fun maps_lookup thy s = Symtab.lookup (MapsData.get thy) s
 
 fun maps_update_thy k minfo = MapsData.map (Symtab.update (k, minfo))