src/HOL/Subst/Unify.thy
changeset 23000 6f158bba99e4
parent 19769 c40ce2de2020
child 24327 a207114007c6
--- a/src/HOL/Subst/Unify.thy	Thu May 17 22:33:41 2007 +0200
+++ b/src/HOL/Subst/Unify.thy	Thu May 17 22:37:34 2007 +0200
@@ -10,8 +10,12 @@
 imports Unifier
 begin
 
-text{*
-Substitution and Unification in Higher-Order Logic.
+subsection {* Substitution and Unification in Higher-Order Logic. *}
+
+text {*
+NB: This theory is already quite old.
+You might want to look at the newer Isar formalization of
+unification in HOL/ex/Unification.thy.
 
 Implements Manna and Waldinger's formalization, with Paulson's simplifications,
 and some new simplifications by Slind.