thys2/Paper/Paper.thy
author Chengsong
Sun, 30 Jan 2022 23:36:31 +0000
changeset 403 6291181fad07
parent 396 cc8e231529fb
child 397 e1b74d618f1b
permissions -rw-r--r--
blexer1 for size bound with strongDB

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

\cite{AusafDyckhoffUrban2016}

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

(*<*)
end
(*>*)