diff -r 9537bf1c4853 -r 5b7a9633cfa8 src/HOL/Imperative_HOL/Heap_Monad.thy --- a/src/HOL/Imperative_HOL/Heap_Monad.thy Sun Nov 02 18:21:14 2014 +0100 +++ b/src/HOL/Imperative_HOL/Heap_Monad.thy Sun Nov 02 18:21:45 2014 +0100 @@ -2,7 +2,7 @@ Author: John Matthews, Galois Connections; Alexander Krauss, Lukas Bulwahn & Florian Haftmann, TU Muenchen *) -header {* A monad with a polymorphic heap and primitive reasoning infrastructure *} +section {* A monad with a polymorphic heap and primitive reasoning infrastructure *} theory Heap_Monad imports