src/HOL/Probability/Lebesgue_Measure.thy
changeset 42067 66c8281349ec
parent 41981 cdf7693bbe08
child 42146 5b52c6a9c627
--- a/src/HOL/Probability/Lebesgue_Measure.thy	Tue Mar 22 18:53:05 2011 +0100
+++ b/src/HOL/Probability/Lebesgue_Measure.thy	Tue Mar 22 20:06:10 2011 +0100
@@ -1,5 +1,10 @@
-(*  Author: Robert Himmelmann, TU Muenchen *)
+(*  Title:      HOL/Probability/Lebesgue_Measure.thy
+    Author:     Johannes Hölzl, TU München
+    Author:     Robert Himmelmann, TU München
+*)
+
 header {* Lebsegue measure *}
+
 theory Lebesgue_Measure
   imports Product_Measure
 begin