diff -r 9537bf1c4853 -r 5b7a9633cfa8 src/HOL/ex/While_Combinator_Example.thy --- a/src/HOL/ex/While_Combinator_Example.thy Sun Nov 02 18:21:14 2014 +0100 +++ b/src/HOL/ex/While_Combinator_Example.thy Sun Nov 02 18:21:45 2014 +0100 @@ -3,7 +3,7 @@ Copyright 2000 TU Muenchen *) -header {* An application of the While combinator *} +section {* An application of the While combinator *} theory While_Combinator_Example imports "~~/src/HOL/Library/While_Combinator"