src/HOL/Library/Convex.thy
changeset 36648 43b66dcd9266
parent 36623 d26348b667f2
child 36778 739a9379e29b
--- a/src/HOL/Library/Convex.thy	Tue May 04 17:53:20 2010 +0200
+++ b/src/HOL/Library/Convex.thy	Tue May 04 18:05:22 2010 +0200
@@ -1,3 +1,10 @@
+(*  Title:      HOL/Library/Convex.thy
+    Author:     Armin Heller, TU Muenchen
+    Author:     Johannes Hoelzl, TU Muenchen
+*)
+
+header {* Convexity in real vector spaces *}
+
 theory Convex
 imports Product_Vector
 begin