Theory Lang
section ‹Imperative Concurrent Language›
text ‹This file defines the syntax and semantics of the concurrent programming language described in
the paper, based on Viktor Vafeiadis' Isabelle soundness proof of CSL~\cite{cslsound},
and adapted to Isabelle 2016-1 by Qin Yu and James Brotherston
(see https://people.mpi-sws.org/~viktor/cslsound/). We also prove some useful lemmas about the semantics.›
theory Lang
imports Main StateModel
begin
subsection ‹Language Syntax and Semantics›
type_synonym state = "store × normal_heap"