src/HOL/Tools/Quotient/quotient_info.ML
changeset 45802 b16f976db515
parent 45534 4ab21521b393
child 46949 94aa7b81bcf6
--- a/src/HOL/Tools/Quotient/quotient_info.ML	Fri Dec 09 16:08:32 2011 +0100
+++ b/src/HOL/Tools/Quotient/quotient_info.ML	Fri Dec 09 18:07:04 2011 +0100
@@ -6,7 +6,7 @@
 
 signature QUOTIENT_INFO =
 sig
-  type quotmaps = {mapfun: string, relmap: string}
+  type quotmaps = {relmap: string}
   val lookup_quotmaps: Proof.context -> string -> quotmaps option
   val lookup_quotmaps_global: theory -> string -> quotmaps option
   val print_quotmaps: Proof.context -> unit
@@ -54,7 +54,7 @@
 (* FIXME just one data slot (record) per program unit *)
 
 (* info about map- and rel-functions for a type *)
-type quotmaps = {mapfun: string, relmap: string}
+type quotmaps = {relmap: string}
 
 structure Quotmaps = Generic_Data
 (
@@ -72,20 +72,18 @@
 val quotmaps_attribute_setup =
   Attrib.setup @{binding map}
     ((Args.type_name false --| Scan.lift (Parse.$$$ "=")) --  (* FIXME Args.type_name true (requires "set" type) *)
-      (Scan.lift (Parse.$$$ "(") |-- Args.const_proper true --| Scan.lift (Parse.$$$ ",") --
-        Args.const_proper true --| Scan.lift (Parse.$$$ ")")) >>
-      (fn (tyname, (mapname, relname)) =>
-        let val minfo = {mapfun = mapname, relmap = relname}
+      Args.const_proper true >>
+      (fn (tyname, relname) =>
+        let val minfo = {relmap = relname}
         in Thm.declaration_attribute (fn _ => Quotmaps.map (Symtab.update (tyname, minfo))) end))
     "declaration of map information"
 
 fun print_quotmaps ctxt =
   let
-    fun prt_map (ty_name, {mapfun, relmap}) =
+    fun prt_map (ty_name, {relmap}) =
       Pretty.block (separate (Pretty.brk 2)
         (map Pretty.str
          ["type:", ty_name,
-          "map:", mapfun,
           "relation map:", relmap]))
   in
     map prt_map (Symtab.dest (Quotmaps.get (Context.Proof ctxt)))