diff -r 9537bf1c4853 -r 5b7a9633cfa8 src/HOL/Proofs/Lambda/ListApplication.thy --- a/src/HOL/Proofs/Lambda/ListApplication.thy Sun Nov 02 18:21:14 2014 +0100 +++ b/src/HOL/Proofs/Lambda/ListApplication.thy Sun Nov 02 18:21:45 2014 +0100 @@ -3,7 +3,7 @@ Copyright 1998 TU Muenchen *) -header {* Application of a term to a list of terms *} +section {* Application of a term to a list of terms *} theory ListApplication imports Lambda begin