src/HOL/Probability/Measure.thy
changeset 45342 5c760e1692b3
parent 44928 7ef6505bde7f
child 45777 c36637603821
--- a/src/HOL/Probability/Measure.thy	Fri Nov 04 17:34:51 2011 +0100
+++ b/src/HOL/Probability/Measure.thy	Fri Nov 04 20:16:42 2011 +0100
@@ -652,7 +652,7 @@
   "almost_everywhere P \<longleftrightarrow> (\<exists>N\<in>null_sets. { x \<in> space M. \<not> P x } \<subseteq> N)"
 
 syntax
-  "_almost_everywhere" :: "'a \<Rightarrow> ('a, 'b) measure_space_scheme \<Rightarrow> ('a \<Rightarrow> bool) \<Rightarrow> bool" ("AE _ in _. _" [0,0,10] 10)
+  "_almost_everywhere" :: "pttrn \<Rightarrow> ('a, 'b) measure_space_scheme \<Rightarrow> bool \<Rightarrow> bool" ("AE _ in _. _" [0,0,10] 10)
 
 translations
   "AE x in M. P" == "CONST measure_space.almost_everywhere M (%x. P)"