diff -r 9537bf1c4853 -r 5b7a9633cfa8 src/HOL/ex/Code_Binary_Nat_examples.thy --- a/src/HOL/ex/Code_Binary_Nat_examples.thy Sun Nov 02 18:21:14 2014 +0100 +++ b/src/HOL/ex/Code_Binary_Nat_examples.thy Sun Nov 02 18:21:45 2014 +0100 @@ -2,7 +2,7 @@ Author: Florian Haftmann, TU Muenchen *) -header {* Simple examples for natural numbers implemented in binary representation. *} +section {* Simple examples for natural numbers implemented in binary representation. *} theory Code_Binary_Nat_examples imports Complex_Main "~~/src/HOL/Library/Code_Binary_Nat"