Paper/Paper.thy
author Christian Urban <urbanc@in.tum.de>
Wed, 17 Mar 2010 20:42:22 +0100
changeset 1491 f970ca9b5bec
parent 1485 c004e7448dca
child 1493 52f68b524fd2
permissions -rw-r--r--
paper uses now a heap file - does not compile so long anymore

(*<*)
theory Paper
imports "../Nominal/Test"
begin
(*>*)

section {* Introduction *}

text {*

  It has not yet fared so well in the POPLmark challenge
  as the second part contain a formalisation of records 
  where ...

  The difficulty can be appreciated by considering that the
  definition given by Leroy in [] is incorrect (it omits a
  side-condition).

  Examples: type-schemes, Spi-calculus

  Contributions:  We provide definitions for when terms
  involving general bindings are alpha-equivelent.
*}

section {* A Brief Overview about the Nominal Logic Work *}

section {* Abstractions *}

section {* Alpha-Equivalence and Free Variables *}



text {*
  Acknowledgements: We thank Andrew Pitts for the many discussions
  about the topic. We thank Peter Sewell for making [] available 
  to us and explaining some of the finer points of the OTT tool.


*}



(*<*)
end
(*>*)