Elimination of fully-functorial style.
authorpaulson
Fri, 16 Feb 1996 13:55:29 +0100
changeset 1505 14f4c55bbe9a
parent 1504 a65cf361e5c1
child 1506 192c48376d25
Elimination of fully-functorial style. Type tactic changed to a type abbrevation (from a datatype). Constructor tactic and function apply deleted.
src/Pure/unify.ML
--- a/src/Pure/unify.ML	Fri Feb 16 13:49:40 1996 +0100
+++ b/src/Pure/unify.ML	Fri Feb 16 13:55:29 1996 +0100
@@ -15,10 +15,7 @@
 
 
 signature UNIFY = 
-sig
-  structure Sign: SIGN
-  structure Envir : ENVIR
-  structure Sequence : SEQUENCE
+  sig
   (*references for control and tracing*)
   val trace_bound: int ref
   val trace_simp: bool ref
@@ -31,20 +28,11 @@
 	-> (Envir.env Sequence.seq)
   val unifiers: Sign.sg * Envir.env * ((term*term)list)
 	-> (Envir.env * (term * term)list) Sequence.seq
-end;
+  end;
 
-functor UnifyFun (structure Sign: SIGN and Envir: ENVIR and Sequence: SEQUENCE
-                  and Pattern:PATTERN
-                  sharing type Sign.sg = Pattern.sg
-                  and     type Envir.env = Pattern.env)
-	: UNIFY = 
+structure Unify	: UNIFY = 
 struct
 
-structure Sign = Sign;
-structure Envir = Envir;
-structure Sequence = Sequence;
-structure Pretty = Sign.Syntax.Pretty;
-
 (*Unification options*)
 
 val trace_bound = ref 10	(*tracing starts above this depth, 0 for full*)
@@ -243,10 +231,10 @@
 
 fun unify_types(T,U, env as Envir.Envir{asol,iTs,maxidx}) =
   if T=U then env
-  else let val (iTs',maxidx') = Sign.Type.unify (#tsig(Sign.rep_sg (!sgr)))
+  else let val (iTs',maxidx') = Type.unify (#tsig(Sign.rep_sg (!sgr)))
                                                 maxidx iTs (U,T)
        in Envir.Envir{asol=asol,maxidx=maxidx',iTs=iTs'} end
-       handle Sign.Type.TUNIFY => raise CANTUNIFY;
+       handle Type.TUNIFY => raise CANTUNIFY;
 
 fun test_unify_types(args as (T,U,_)) =
 let val sot = Sign.string_of_typ (!sgr);