src/HOL/Probability/Finite_Product_Measure.thy
changeset 61378 3e04c9ca001a
parent 61363 76ac925927aa
child 61424 c3658c18b7bc
--- a/src/HOL/Probability/Finite_Product_Measure.thy	Fri Oct 09 19:51:20 2015 +0200
+++ b/src/HOL/Probability/Finite_Product_Measure.thy	Fri Oct 09 20:26:03 2015 +0200
@@ -170,13 +170,8 @@
 
 syntax
   "_PiM" :: "pttrn \<Rightarrow> 'i set \<Rightarrow> 'a measure \<Rightarrow> ('i => 'a) measure"  ("(3PIM _:_./ _)" 10)
-
 syntax (xsymbols)
   "_PiM" :: "pttrn \<Rightarrow> 'i set \<Rightarrow> 'a measure \<Rightarrow> ('i => 'a) measure"  ("(3\<Pi>\<^sub>M _\<in>_./ _)"  10)
-
-syntax (HTML output)
-  "_PiM" :: "pttrn \<Rightarrow> 'i set \<Rightarrow> 'a measure \<Rightarrow> ('i => 'a) measure"  ("(3\<Pi>\<^sub>M _\<in>_./ _)"  10)
-
 translations
   "PIM x:I. M" == "CONST PiM I (%x. M)"