Theory MLSS_Suc_Theory
theory MLSS_Suc_Theory
imports Main "HOL-Library.Adhoc_Overloading" Fresh_Identifiers.Fresh
begin
section ‹Solver for the Theory of the Successor Function›
text ‹
This theory implements a solver for the theory consisting of
variables, 0, and the successor function.
We only deal with equality and not with disequality or inequality.
Disequalities of the form \<^term>‹l ≠ 0› are translated to
\<^term>‹l = Suc x› for some fresh \<^term>‹x›.
Note that disequalities and inequalities can always be fulfilled
by choosing large enough values for the variables.
›