diff -r 0baae4311a9f -r b9556a055632 src/HOL/Library/ListVector.thy --- a/src/HOL/Library/ListVector.thy Sun Nov 02 17:16:01 2014 +0100 +++ b/src/HOL/Library/ListVector.thy Sun Nov 02 17:20:45 2014 +0100 @@ -1,6 +1,6 @@ (* Author: Tobias Nipkow, 2007 *) -header {* Lists as vectors *} +section {* Lists as vectors *} theory ListVector imports List Main