Fun-Paper/Paper.thy
author Christian Urban <urbanc@in.tum.de>
Tue, 05 Jul 2011 15:00:41 +0200
changeset 2946 d9c3cc271e62
parent 2931 aaef9dec5e1d
permissions -rw-r--r--
added a tactic "all_trivials" which simplifies all trivial constructor cases and leaves the others untouched.

(*<*)
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
(*>*)