diff -r 4e796867ccb5 -r a4e69ce247e0 src/HOL/Nominal/Examples/Weakening.thy --- a/src/HOL/Nominal/Examples/Weakening.thy Mon Dec 31 19:36:29 2007 +0100 +++ b/src/HOL/Nominal/Examples/Weakening.thy Tue Jan 01 07:28:20 2008 +0100 @@ -4,11 +4,11 @@ imports "../Nominal" begin -section {* Weakening Example for the Simply-Typed Lambda-Calculus *} +section {* Weakening Property in the Simply-Typed Lambda-Calculus *} atom_decl name -text {* Terms and types *} +text {* Terms and Types *} nominal_datatype lam = Var "name" | App "lam" "lam" @@ -48,7 +48,7 @@ text {* We derive the strong induction principle for the typing relation (this induction principle has the variable convention - already built in). + already built-in). *} equivariance typing nominal_inductive typing @@ -144,6 +144,7 @@ oops text{* The complete proof without using the variable convention. *} + lemma weakening_with_explicit_renaming: fixes \1 \2::"(name\ty) list" assumes a: "\1 \ t : T" @@ -189,9 +190,9 @@ qed (auto) text {* - Compare the proof with explicit renamings to version1 and version2, - and imagine you are proving something more substantial than the - weakening lemma. + Moral: compare the proof with explicit renamings to version1 and version2, + and imagine you are proving something more substantial than the weakening + lemma. *} end \ No newline at end of file