src/HOL/Imperative_HOL/ex/Subarray.thy
changeset 36098 53992c639da5
parent 30689 b14b2cc4e25e
child 37719 271ecd4fb9f9
--- a/src/HOL/Imperative_HOL/ex/Subarray.thy	Wed Apr 07 22:22:49 2010 +0200
+++ b/src/HOL/Imperative_HOL/ex/Subarray.thy	Thu Apr 08 08:17:27 2010 +0200
@@ -1,3 +1,9 @@
+(*  Title:      HOL/Imperative_HOL/ex/Subarray.thy
+    Author:     Lukas Bulwahn, TU Muenchen
+*)
+
+header {* Theorems about sub arrays *}
+
 theory Subarray
 imports Array Sublist
 begin