thys/Paper/Paper.thy
changeset 95 a33d3040bf7e
child 97 38696f516c6b
equal deleted inserted replaced
94:5b01f7c233f8 95:a33d3040bf7e
       
     1 (*<*)
       
     2 theory Paper
       
     3 imports "../ReStar" "~~/src/HOL/Library/LaTeXsugar"
       
     4 begin
       
     5 (*>*)
       
     6 
       
     7 section {* Introduction *}
       
     8 
       
     9  
       
    10 
       
    11 text {*
       
    12   %\noindent
       
    13   %{\bf Acknowledgements:}
       
    14   %We are grateful for the comments we received from anonymous
       
    15   %referees.
       
    16 
       
    17   \bibliographystyle{plain}
       
    18   \bibliography{root}
       
    19 *}
       
    20 
       
    21 
       
    22 (*<*)
       
    23 end
       
    24 (*>*)