Fun-Paper/Paper.thy
author Christian Urban <urbanc@in.tum.de>
Mon, 04 Jun 2012 21:39:51 +0100
changeset 3183 313e6f2cdd89
parent 2931 aaef9dec5e1d
permissions -rw-r--r--
added permutation simplification to the simplifier; this makes the simplifier more powerful, but it potentially loops more often

(*<*)
theory Paper
imports "~~/src/HOL/Library/LaTeXsugar" 
begin

declare [[show_question_marks = false]]

section {* Introduction *}

text {*
mention Russo paper which concludes that technology is not 
ready beyond core-calculi.



*}


(*<*)
end
(*>*)