Theory Lam_ml
section ‹Introduction›
theory Lam_ml
imports "HOL-Nominal.Nominal" "HOL-Library.LaTeXsugar"
begin
text_raw ‹\label{chap:formal}›
text ‹This article contains a formalization of the strong normalization
theorem for the $\lambda_{ml}$-calculus. The formalization is based on a proof
by Lindley and Stark \<^cite>‹"TT-lifting"›. An informal description of the
formalization can be found in \<^cite>‹"Doczkal:09"›.
This formalization extends the example proof of strong normalization for the
simply-typed $\lambda$-calculus, which is included in the Isabelle distribution
\<^cite>‹"SN.thy"›. The parts of the original proof which have been left unchanged
are not displayed in this document.
The next section deals with the formalization of syntax, typing, and
substitution. Section~\ref{sec:reduction} contains the formalization of the
reduction relation. Section~\ref{sec:stacks} defines stacks which are used to
define the reducibility relation in Section~\ref{sec:reducibility-formal}. The
following sections contain proofs about the reducibility relation, ending with
the normalization theorem in Section~\ref{sec:FTLR}.›
section ‹The Calculus›
text_raw ‹\label{sec:calc}›