Theory HOL-ex.Unification
section ‹Substitution and Unification›
theory Unification
imports Main
begin
text ‹
Implements Manna \& Waldinger's formalization, with Paulson's
simplifications, and some new simplifications by Slind and Krauss.
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
K Slind, Reasoning about Terminating Functional Programs,
Ph.D. thesis, TUM, 1999, Sect. 5.8
A Krauss, Partial and Nested Recursive Function Definitions in
Higher-Order Logic, JAR 44(4):303-336, 2010. Sect. 6.3
›
subsection ‹Terms›
text ‹Binary trees with leaves that are constants or variables.›