src/HOL/Hoare/Pointer_ExamplesAbort.thy
changeset 72990 db8f94656024
parent 71989 bad75618fb82
--- a/src/HOL/Hoare/Pointer_ExamplesAbort.thy	Wed Dec 23 21:32:24 2020 +0100
+++ b/src/HOL/Hoare/Pointer_ExamplesAbort.thy	Wed Dec 23 22:25:22 2020 +0100
@@ -1,15 +1,17 @@
 (*  Title:      HOL/Hoare/Pointer_ExamplesAbort.thy
     Author:     Tobias Nipkow
     Copyright   2002 TUM
-
-Examples of verifications of pointer programs
 *)
 
-theory Pointer_ExamplesAbort imports HeapSyntaxAbort begin
+section \<open>Examples of verifications of pointer programs\<close>
 
-section "Verifications"
+theory Pointer_ExamplesAbort
+  imports HeapSyntaxAbort
+begin
 
-subsection "List reversal"
+subsection "Verifications"
+
+subsubsection "List reversal"
 
 text "Interestingly, this proof is the same as for the unguarded program:"