moved specific map_typ/term to sign.ML;
authorwenzelm
Thu, 02 Feb 2006 12:52:18 +0100
changeset 18893 2dbf73278b0e
parent 18892 51360da418b2
child 18894 9c8c60853966
moved specific map_typ/term to sign.ML;
src/Pure/term.ML
--- a/src/Pure/term.ML	Thu Feb 02 12:52:16 2006 +0100
+++ b/src/Pure/term.ML	Thu Feb 02 12:52:18 2006 +0100
@@ -194,8 +194,6 @@
   val maxidx_typs: typ list -> int -> int
   val maxidx_term: term -> int -> int
   val invent_names: string list -> string -> int -> string list
-  val map_typ: (string -> string) -> (string -> string) -> typ -> typ
-  val map_term: (string -> string) -> (string -> string) -> (string -> string) -> term -> term
   val dest_abs: string * typ * term -> string * term
   val bound: int -> string
   val is_bound: string -> bool
@@ -1124,19 +1122,6 @@
 
 fun exists_Const P = exists_subterm (fn Const c => P c | _ => false);
 
-(*map classes, tycons*)
-fun map_typ f g (Type (c, Ts)) = Type (g c, map (map_typ f g) Ts)
-  | map_typ f _ (TFree (x, S)) = TFree (x, map f S)
-  | map_typ f _ (TVar (xi, S)) = TVar (xi, map f S);
-
-(*map classes, tycons, consts*)
-fun map_term f g h (Const (c, T)) = Const (h c, map_typ f g T)
-  | map_term f g _ (Free (x, T)) = Free (x, map_typ f g T)
-  | map_term f g _ (Var (xi, T)) = Var (xi, map_typ f g T)
-  | map_term _ _ _ (t as Bound _) = t
-  | map_term f g h (Abs (x, T, t)) = Abs (x, map_typ f g T, map_term f g h t)
-  | map_term f g h (t $ u) = map_term f g h t $ map_term f g h u;
-
 
 (** TFrees and TVars **)