diff -r cbd6a709a664 -r 471308f23649 Paper/Paper.thy --- a/Paper/Paper.thy Tue Mar 30 09:00:52 2010 +0200 +++ b/Paper/Paper.thy Tue Mar 30 09:15:40 2010 +0200 @@ -1090,7 +1090,8 @@ \noindent We define them together with the auxiliary free variable functions for - binding functions + binding functions. Given binding functions of types + @{text "bn\<^isub>1 :: ty\<^isub>i\<^isub>1 \ \ \ bn\<^isub>m :: ty\<^isub>i\<^isub>m \ \"} we need to define \begin{center} @{text "fv_bn\<^isub>1 :: ty\<^isub>i\<^isub>1 \ atom set \ fv_bn\<^isub>m :: ty\<^isub>i\<^isub>m \ atom set"} @@ -1167,6 +1168,23 @@ \end{tabular} \end{center} + We then define the alpha equivalence relations. For the types @{text "ty\<^isub>1, \, ty\<^isub>n"} + we need to define + + \begin{center} + @{text "\\<^isub>1 :: ty\<^isub>1 \ ty\<^isub>1 \ bool \ \\<^isub>n :: ty\<^isub>n \ ty\<^isub>n \ bool"} + \end{center} + + \noindent + together with the auxiliary equivalences for binding functions. Given binding + functions for types @{text "bn\<^isub>1 :: ty\<^isub>i\<^isub>1 \ \ \ bn\<^isub>m :: ty\<^isub>i\<^isub>m \ \"} we need to define + \begin{center} + @{text "\bn\<^isub>1 :: ty\<^isub>i\<^isub>1 \ ty\<^isub>i\<^isub>1 \ bool \ \bn\<^isub>n :: ty\<^isub>i\<^isub>m \ ty\<^isub>i\<^isub>m \ bool"} + \end{center} + + + + *} section {* The Lifting of Definitions and Properties *}