src/HOL/Hoare/Pointer_Examples.thy
changeset 41959 b460124855b8
parent 38353 d98baa2cf589
child 44890 22f665a2e91c
--- a/src/HOL/Hoare/Pointer_Examples.thy	Sun Mar 13 22:24:10 2011 +0100
+++ b/src/HOL/Hoare/Pointer_Examples.thy	Sun Mar 13 22:55:50 2011 +0100
@@ -1,8 +1,8 @@
-(*  Title:      HOL/Hoare/Pointers.thy
+(*  Title:      HOL/Hoare/Pointer_Examples.thy
     Author:     Tobias Nipkow
     Copyright   2002 TUM
 
-Examples of verifications of pointer programs
+Examples of verifications of pointer programs.
 *)
 
 theory Pointer_Examples imports HeapSyntax begin