renamed transfer to transform (Markus)
authorChristian Urban <urbanc@in.tum.de>
Thu, 31 Dec 2009 23:53:10 +0100
changeset 799 0755f8fd56b3
parent 798 a422a51bb0eb
child 800 71225f4a4635
renamed transfer to transform (Markus)
Quot/quotient_def.ML
Quot/quotient_info.ML
Quot/quotient_typ.ML
--- a/Quot/quotient_def.ML	Wed Dec 30 12:10:57 2009 +0000
+++ b/Quot/quotient_def.ML	Thu Dec 31 23:53:10 2009 +0100
@@ -44,7 +44,7 @@
 
   val ((trm, thm), lthy') = define qconst_bname mx attr newrhs lthy
 
-  fun qcinfo phi = qconsts_transfer phi {qconst = trm, rconst = rhs, def = thm}
+  fun qcinfo phi = transform_qconsts phi {qconst = trm, rconst = rhs, def = thm}
   val lthy'' = Local_Theory.declaration true
                  (fn phi => qconsts_update_gen lhs_str (qcinfo phi)) lthy'
 in
--- a/Quot/quotient_info.ML	Wed Dec 30 12:10:57 2009 +0000
+++ b/Quot/quotient_info.ML	Thu Dec 31 23:53:10 2009 +0100
@@ -9,14 +9,14 @@
   val print_mapsinfo: Proof.context -> unit
 
   type quotdata_info = {qtyp: typ, rtyp: typ, equiv_rel: term, equiv_thm: thm}
-  val quotdata_transfer: morphism -> quotdata_info -> quotdata_info
+  val transform_quotdata: morphism -> quotdata_info -> quotdata_info
   val quotdata_lookup: theory -> string -> quotdata_info     (* raises NotFound *)
   val quotdata_update_thy: string -> quotdata_info -> theory -> theory
   val quotdata_update_gen: string -> quotdata_info -> Context.generic -> Context.generic
   val print_quotinfo: Proof.context -> unit
 
   type qconsts_info = {qconst: term, rconst: term, def: thm}
-  val qconsts_transfer: morphism -> qconsts_info -> qconsts_info
+  val transform_qconsts: morphism -> qconsts_info -> qconsts_info
   val qconsts_lookup: theory -> term -> qconsts_info     (* raises NotFound *)
   val qconsts_update_thy: string -> qconsts_info -> theory -> theory
   val qconsts_update_gen: string -> qconsts_info -> Context.generic -> Context.generic
@@ -138,7 +138,7 @@
    val extend = I
    val merge = Symtab.merge (K true)) 
 
-fun quotdata_transfer phi {qtyp, rtyp, equiv_rel, equiv_thm} =
+fun transform_quotdata phi {qtyp, rtyp, equiv_rel, equiv_thm} =
     {qtyp = Morphism.typ phi qtyp,
      rtyp = Morphism.typ phi rtyp,
      equiv_rel = Morphism.term phi equiv_rel,
@@ -185,7 +185,7 @@
    val extend = I
    val merge = Symtab.merge (K true))
 
-fun qconsts_transfer phi {qconst, rconst, def} =
+fun transform_qconsts phi {qconst, rconst, def} =
     {qconst = Morphism.term phi qconst,
      rconst = Morphism.term phi rconst,
      def = Morphism.thm phi def}
--- a/Quot/quotient_typ.ML	Wed Dec 30 12:10:57 2009 +0000
+++ b/Quot/quotient_typ.ML	Thu Dec 31 23:53:10 2009 +0100
@@ -154,7 +154,7 @@
 
   (* storing the quot-info *)
   (* FIXME: VarifyT should not be used - at the moment it allows matching against the types. *)
-  fun qinfo phi = quotdata_transfer phi
+  fun qinfo phi = transform_quotdata phi
                     {qtyp = Logic.varifyT Abs_ty, rtyp = Logic.varifyT rty, 
                      equiv_rel = map_types Logic.varifyT rel, equiv_thm = equiv_thm}
   val lthy4 = Local_Theory.declaration true