thys2/Paper/Paper.thy
changeset 396 cc8e231529fb
child 397 e1b74d618f1b
--- /dev/null	Thu Jan 01 00:00:00 1970 +0000
+++ b/thys2/Paper/Paper.thy	Tue Jan 25 13:12:50 2022 +0000
@@ -0,0 +1,21 @@
+(*<*)
+theory Paper
+imports 
+   "../Lexer"
+   "../Simplifying" 
+   "../Positions"
+   "../SizeBound4" 
+   "HOL-Library.LaTeXsugar"
+begin
+(*>*)
+text {*
+
+\cite{AusafDyckhoffUrban2016}
+
+%%\bibliographystyle{plain}
+\bibliography{root}
+*}
+
+(*<*)
+end
+(*>*)
\ No newline at end of file