Fun-Paper/Paper.thy
author Cezary Kaliszyk <kaliszyk@in.tum.de>
Sat, 02 Jul 2011 12:40:59 +0900
changeset 2932 e8ab80062061
parent 2931 aaef9dec5e1d
permissions -rw-r--r--
Did the proofs of height and subst for Let with list-like binders. Having apply_assns allows proving things by alpha_bn

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