src/HOL/Analysis/Finite_Product_Measure.thy
changeset 80768 c7723cc15de8
parent 78516 56a408fa2440
child 80914 d97fdabd9e2b
--- a/src/HOL/Analysis/Finite_Product_Measure.thy	Sun Aug 25 20:54:20 2024 +0200
+++ b/src/HOL/Analysis/Finite_Product_Measure.thy	Sun Aug 25 21:10:01 2024 +0200
@@ -170,6 +170,8 @@
 
 syntax
   "_PiM" :: "pttrn \<Rightarrow> 'i set \<Rightarrow> 'a measure \<Rightarrow> ('i => 'a) measure"  ("(3\<Pi>\<^sub>M _\<in>_./ _)"  10)
+syntax_consts
+  "_PiM" == PiM
 translations
   "\<Pi>\<^sub>M x\<in>I. M" == "CONST PiM I (%x. M)"