Theory OpSem
section ‹Logical relations for computational adequacy›
theory OpSem
imports
Basis
PCF
begin
text‹
\label{sec:opsem}
We relate the denotational semantics for PCF of \S\ref{sec:densem} to
a \emph{big-step} (or \emph{natural}) operational semantics. This
follows \<^citet>‹"DBLP:conf/mfps/Pitts93"›.
›
subsection‹Direct semantics using de Bruijn notation›
text‹
\label{sec:directsem_db}
In contrast to \S\ref{sec:directsem} we must be more careful in our
treatment of ‹α›-equivalent terms, as we would like our
operational semantics to identify of all these. To that end we adopt
de Bruijn notation, adapting the work of
\<^citet>‹"DBLP:journals/jar/Nipkow01"›, and show that it is suitably
equivalent to our original syntactic story.
›