thys2/Paper/Paper.thy
author Christian Urban <christian.urban@kcl.ac.uk>
Tue, 25 Jan 2022 13:12:50 +0000
changeset 396 cc8e231529fb
child 397 e1b74d618f1b
permissions -rw-r--r--
added ITP paper

(*<*)
theory Paper
imports 
   "../Lexer"
   "../Simplifying" 
   "../Positions"
   "../SizeBound4" 
   "HOL-Library.LaTeXsugar"
begin
(*>*)
text {*

\cite{AusafDyckhoffUrban2016}

%%\bibliographystyle{plain}
\bibliography{root}
*}

(*<*)
end
(*>*)