src/HOL/Subst/ROOT.ML
changeset 3192 a75558a4ed37
parent 1465 5d7a7e439cec
child 6349 f7750d816c21
--- a/src/HOL/Subst/ROOT.ML	Thu May 15 12:29:59 1997 +0200
+++ b/src/HOL/Subst/ROOT.ML	Thu May 15 12:40:01 1997 +0200
@@ -1,32 +1,34 @@
 (*  Title:      HOL/Subst/ROOT.ML
     ID:         $Id$
-    Author:     Martin Coen, Cambridge University Computer Laboratory
-    Copyright   1993  University of Cambridge
+    Authors:     Martin Coen, Cambridge University Computer Laboratory
+                 Konrad Slind, TU Munich
+    Copyright   1993  University of Cambridge,
+                1996  TU Munich
 
 Substitution and Unification in Higher-Order Logic. 
 
-Implements Manna & Waldinger's formalization, with Paulson's simplifications:
+Implements Manna & Waldinger's formalization, with Paulson's simplifications,
+and some new simplifications by Slind.
 
 Z Manna & R Waldinger, Deductive Synthesis of the Unification Algorithm. 
 SCP 1 (1981), 5-48
 
 L C Paulson, Verifying the Unification Algorithm in LCF. SCP 5 (1985), 143-170
 
-setplus      -  minor additions to HOL's set theory
-alist        -  association lists
-uterm        -  inductive data type of terms
-utlemmas     -  definition of occurs and vars_of for terms
-subst        -  substitutions
-unifier      -  specification of unification and conditions for 
+AList        -  association lists
+UTerm        -  data type of terms
+Subst        -  substitutions
+Unifier      -  specification of unification and conditions for 
                 correctness and termination
+Unify        -  the unification function
 
-To load, go to the parent directory and type use"Subst/ROOT.ML";
+To load, type use"ROOT.ML"; into an Isabelle-HOL that has TFL 
+also loaded. 
 *)
 
 HOL_build_completed;    (*Cause examples to fail if HOL did*)
 
 writeln"Root file for Substitutions and Unification";
-
-use_thy "Unifier";
+use_thy "Unify";
 
 writeln"END: Root file for Substitutions and Unification";