Quotient-Paper/Paper.thy
author Christian Urban <urbanc@in.tum.de>
Thu, 29 Apr 2010 09:13:18 +0200
changeset 1975 b1281a0051ae
child 1978 8feedc0d4ea8
permissions -rw-r--r--
added stub for quotient paper; call with isabelle make qpaper

(*<*)
theory Paper
imports "Quotient" 
        "LaTeXsugar"
begin
(*>*)

section {* Introduction *}

text {* TBD *}



(*<*)
end
(*>*)