diff -r 8ad8d02b973f -r e56aedec11f3 src/Pure/term.ML --- a/src/Pure/term.ML Fri Mar 01 22:28:59 2002 +0100 +++ b/src/Pure/term.ML Fri Mar 01 22:30:01 2002 +0100 @@ -36,6 +36,7 @@ Abs of string * typ * term | $ of term * term structure Vartab : TABLE + structure Typtab : TABLE structure Termtab : TABLE exception TYPE of string * typ list * term list exception TERM of string * term list @@ -215,16 +216,16 @@ (*Terms. Bound variables are indicated by depth number. Free variables, (scheme) variables and constants have names. An term is "closed" if every bound variable of level "lev" - is enclosed by at least "lev" abstractions. + is enclosed by at least "lev" abstractions. It is possible to create meaningless terms containing loose bound vars or type mismatches. But such terms are not allowed in rules. *) -datatype term = +datatype term = Const of string * typ - | Free of string * typ + | Free of string * typ | Var of indexname * typ | Bound of int | Abs of string*typ*term @@ -310,18 +311,18 @@ Ts = [T0,T1,...] holds types of bound variables 0, 1, ...*) fun type_of1 (Ts, Const (_,T)) = T | type_of1 (Ts, Free (_,T)) = T - | type_of1 (Ts, Bound i) = (nth_elem (i,Ts) + | type_of1 (Ts, Bound i) = (nth_elem (i,Ts) handle LIST _ => raise TYPE("type_of: bound variable", [], [Bound i])) | type_of1 (Ts, Var (_,T)) = T | type_of1 (Ts, Abs (_,T,body)) = T --> type_of1(T::Ts, body) - | type_of1 (Ts, f$u) = + | type_of1 (Ts, f$u) = let val U = type_of1(Ts,u) and T = type_of1(Ts,f) in case T of Type("fun",[T1,T2]) => if T1=U then T2 else raise TYPE ("type_of: type mismatch in application", [T1,U], [f$u]) - | _ => raise TYPE + | _ => raise TYPE ("type_of: function type is expected in application", [T,U], [f$u]) end; @@ -329,7 +330,7 @@ fun type_of t : typ = type_of1 ([],t); (*Determines the type of a term, with minimal checking*) -fun fastype_of1 (Ts, f$u) = +fun fastype_of1 (Ts, f$u) = (case fastype_of1 (Ts,f) of Type("fun",[_,T]) => T | _ => raise TERM("fastype_of: expected function type", [f$u])) @@ -337,7 +338,7 @@ | fastype_of1 (_, Free (_,T)) = T | fastype_of1 (Ts, Bound i) = (nth_elem(i,Ts) handle LIST _ => raise TERM("fastype_of: Bound", [Bound i])) - | fastype_of1 (_, Var (_,T)) = T + | fastype_of1 (_, Var (_,T)) = T | fastype_of1 (Ts, Abs (_,T,u)) = T --> fastype_of1 (T::Ts, u); fun fastype_of t : typ = fastype_of1 ([],t); @@ -346,11 +347,11 @@ val list_abs = foldr (fn ((x, T), t) => Abs (x, T, t)); (* maps (x1,...,xn)t to t *) -fun strip_abs_body (Abs(_,_,t)) = strip_abs_body t +fun strip_abs_body (Abs(_,_,t)) = strip_abs_body t | strip_abs_body u = u; (* maps (x1,...,xn)t to [x1, ..., xn] *) -fun strip_abs_vars (Abs(a,T,t)) = (a,T) :: strip_abs_vars t +fun strip_abs_vars (Abs(a,T,t)) = (a,T) :: strip_abs_vars t | strip_abs_vars u = [] : (string*typ) list; @@ -370,9 +371,9 @@ (* maps f(t1,...,tn) to (f, [t1,...,tn]) ; naturally tail-recursive*) -fun strip_comb u : term * term list = +fun strip_comb u : term * term list = let fun stripc (f$t, ts) = stripc (f, t::ts) - | stripc x = x + | stripc x = x in stripc(u,[]) end; @@ -434,22 +435,22 @@ fun flexpair T = Const("=?=", T-->T-->propT); (* maps !!x1...xn. t to t *) -fun strip_all_body (Const("all",_)$Abs(_,_,t)) = strip_all_body t +fun strip_all_body (Const("all",_)$Abs(_,_,t)) = strip_all_body t | strip_all_body t = t; (* maps !!x1...xn. t to [x1, ..., xn] *) fun strip_all_vars (Const("all",_)$Abs(a,T,t)) = - (a,T) :: strip_all_vars t + (a,T) :: strip_all_vars t | strip_all_vars t = [] : (string*typ) list; (*increments a term's non-local bound variables required when moving a term within abstractions inc is increment for bound variables lev is level at which a bound variable is considered 'loose'*) -fun incr_bv (inc, lev, u as Bound i) = if i>=lev then Bound(i+inc) else u +fun incr_bv (inc, lev, u as Bound i) = if i>=lev then Bound(i+inc) else u | incr_bv (inc, lev, Abs(a,T,body)) = Abs(a, T, incr_bv(inc,lev+1,body)) - | incr_bv (inc, lev, f$t) = + | incr_bv (inc, lev, f$t) = incr_bv(inc,lev,f) $ incr_bv(inc,lev,t) | incr_bv (inc, lev, u) = u; @@ -478,11 +479,11 @@ (*Accumulate all 'loose' bound vars referring to level 'lev' or beyond. (Bound 0) is loose at level 0 *) -fun add_loose_bnos (Bound i, lev, js) = +fun add_loose_bnos (Bound i, lev, js) = if i=n are reduced by "n" to compensate for the disappearance of lambdas. *) -fun subst_bounds (args: term list, t) : term = +fun subst_bounds (args: term list, t) : term = let val n = length args; fun subst (t as Bound i, lev) = (if i t | _ => subst (t,0) end; (*Special case: one argument*) -fun subst_bound (arg, t) : term = +fun subst_bound (arg, t) : term = let fun subst (t as Bound i, lev) = if it) | subst_free pairs = - let fun substf u = + let fun substf u = case gen_assoc (op aconv) (pairs, u) of Some u' => u' | None => (case u of Abs(a,T,t) => Abs(a, T, substf t) @@ -634,7 +635,7 @@ fun xless ((a,i), (b,j): indexname) = i string_ord (x, y) | ord => ord); +val sort_ord = list_ord string_ord; + (* typ_ord *) -(*assumes that TFrees / TVars with the same name have same sorts*) -fun typ_ord (Type (a, Ts), Type (b, Us)) = - (case string_ord (a, b) of EQUAL => typs_ord (Ts, Us) | ord => ord) +fun typ_ord (Type x, Type y) = prod_ord string_ord typs_ord (x, y) | typ_ord (Type _, _) = GREATER | typ_ord (TFree _, Type _) = LESS - | typ_ord (TFree (a, _), TFree (b, _)) = string_ord (a, b) + | typ_ord (TFree x, TFree y) = prod_ord string_ord sort_ord (x, y) | typ_ord (TFree _, TVar _) = GREATER | typ_ord (TVar _, Type _) = LESS | typ_ord (TVar _, TFree _) = LESS - | typ_ord (TVar (xi, _), TVar (yj, _)) = indexname_ord (xi, yj) + | typ_ord (TVar x, TVar y) = prod_ord indexname_ord sort_ord (x, y) and typs_ord Ts_Us = list_ord typ_ord Ts_Us; @@ -1027,6 +1028,7 @@ fun termless tu = (term_ord tu = LESS); structure Vartab = TableFun(type key = indexname val ord = indexname_ord); +structure Typtab = TableFun(type key = typ val ord = typ_ord); structure Termtab = TableFun(type key = term val ord = term_ord); (*Substitute for type Vars in a type, version using Vartab*) @@ -1041,72 +1043,33 @@ val subst_TVars_Vartab = map_term_types o typ_subst_TVars_Vartab; -(*** Compression of terms and types by sharing common subtrees. - Saves 50-75% on storage requirements. As it is fairly slow, - it is called only for axioms, stored theorems, etc. ***) +(*** Compression of terms and types by sharing common subtrees. + Saves 50-75% on storage requirements. As it is a bit slow, + it should be called only for axioms, stored theorems, etc. + Recorded term and type fragments are never disposed. ***) (** Sharing of types **) -fun atomic_tag (Type (a,_)) = if a<>"fun" then a else raise Match - | atomic_tag (TFree (a,_)) = a - | atomic_tag (TVar ((a,_),_)) = a; - -fun type_tag (Type("fun",[S,T])) = atomic_tag S ^ type_tag T - | type_tag T = atomic_tag T; - -val memo_types = ref (Symtab.empty : typ list Symtab.table); - -(* special case of library/find_first *) -fun find_type (T, []: typ list) = None - | find_type (T, T'::Ts) = - if T=T' then Some T' - else find_type (T, Ts); +val memo_types = ref (Typtab.empty: typ Typtab.table); fun compress_type T = - let val tag = type_tag T - val tylist = Symtab.lookup_multi (!memo_types, tag) - in - case find_type (T,tylist) of - Some T' => T' - | None => - let val T' = - case T of - Type (a,Ts) => Type (a, map compress_type Ts) - | _ => T - in memo_types := Symtab.update ((tag, T'::tylist), !memo_types); - T - end - end - handle Match => - let val Type (a,Ts) = T - in Type (a, map compress_type Ts) end; + (case Typtab.lookup (! memo_types, T) of + Some T' => T' + | None => + let val T' = (case T of Type (a, Ts) => Type (a, map compress_type Ts) | _ => T) + in memo_types := Typtab.update ((T', T'), ! memo_types); T' end); + (** Sharing of atomic terms **) -val memo_terms = ref (Symtab.empty : term list Symtab.table); - -(* special case of library/find_first *) -fun find_term (t, []: term list) = None - | find_term (t, t'::ts) = - if t=t' then Some t' - else find_term (t, ts); - -fun const_tag (Const (a,_)) = a - | const_tag (Free (a,_)) = a - | const_tag (Var ((a,i),_)) = a - | const_tag (t as Bound _) = ".B."; +val memo_terms = ref (Termtab.empty : term Termtab.table); fun share_term (t $ u) = share_term t $ share_term u - | share_term (Abs (a,T,u)) = Abs (a, T, share_term u) + | share_term (Abs (a, T, u)) = Abs (a, T, share_term u) | share_term t = - let val tag = const_tag t - val ts = Symtab.lookup_multi (!memo_terms, tag) - in - case find_term (t,ts) of - Some t' => t' - | None => (memo_terms := Symtab.update ((tag, t::ts), !memo_terms); - t) - end; + (case Termtab.lookup (! memo_terms, t) of + Some t' => t' + | None => (memo_terms := Termtab.update ((t, t), ! memo_terms); t)); val compress_term = share_term o map_term_types compress_type;