src/HOL/Probability/Information.thy
changeset 41413 64cd30d6b0b8
parent 41095 c335d880ff82
child 41661 baf1964bc468
--- a/src/HOL/Probability/Information.thy	Wed Dec 29 13:51:17 2010 +0100
+++ b/src/HOL/Probability/Information.thy	Wed Dec 29 17:34:41 2010 +0100
@@ -1,5 +1,8 @@
 theory Information
-imports Probability_Space Convex Lebesgue_Measure
+imports
+  Probability_Space
+  "~~/src/HOL/Library/Convex"
+  Lebesgue_Measure
 begin
 
 lemma log_le: "1 < a \<Longrightarrow> 0 < x \<Longrightarrow> x \<le> y \<Longrightarrow> log a x \<le> log a y"