src/HOL/Analysis/Set_Integral.thy
changeset 63958 02de4a58e210
parent 63941 f353674c2528
child 64283 979cdfdf7a79
--- a/src/HOL/Analysis/Set_Integral.thy	Thu Sep 29 13:02:43 2016 +0200
+++ b/src/HOL/Analysis/Set_Integral.thy	Thu Sep 29 13:54:57 2016 +0200
@@ -27,16 +27,6 @@
 translations
 "LINT x:A|M. f" == "CONST set_lebesgue_integral M A (\<lambda>x. f)"
 
-abbreviation
-  "set_almost_everywhere A M P \<equiv> AE x in M. x \<in> A \<longrightarrow> P x"
-
-syntax
-  "_set_almost_everywhere" :: "pttrn \<Rightarrow> 'a set \<Rightarrow> 'a \<Rightarrow> bool \<Rightarrow> bool"
-("AE _\<in>_ in _./ _" [0,0,0,10] 10)
-
-translations
-  "AE x\<in>A in M. P" == "CONST set_almost_everywhere A M (\<lambda>x. P)"
-
 (*
     Notation for integration wrt lebesgue measure on the reals: