diff -r 3e3e7a68cd80 -r 6ad2c917dd2e src/HOL/Probability/Fin_Map.thy --- a/src/HOL/Probability/Fin_Map.thy Wed Oct 09 22:01:33 2024 +0200 +++ b/src/HOL/Probability/Fin_Map.thy Wed Oct 09 23:38:29 2024 +0200 @@ -13,7 +13,7 @@ stay close to the developments of (finite) products \<^const>\Pi\<^sub>E\ and their sigma-algebra \<^const>\Pi\<^sub>M\.\ -type_notation fmap (\(_ \\<^sub>F /_)\ [22, 21] 21) +type_notation fmap (\(\notation=\infix fmap\\_ \\<^sub>F /_)\ [22, 21] 21) unbundle fmap.lifting @@ -25,7 +25,8 @@ lemma finite_domain[simp, intro]: "finite (domain P)" by transfer simp -lift_definition proj :: "('i \\<^sub>F 'a) \ 'i \ 'a" (\'((_)')\<^sub>F\ [0] 1000) is +lift_definition proj :: "('i \\<^sub>F 'a) \ 'i \ 'a" + (\(\indent=1 notation=\mixfix proj\\'(_')\<^sub>F)\ [0] 1000) is "\f x. if x \ dom f then the (f x) else undefined" . declare [[coercion proj]] @@ -89,7 +90,8 @@ "Pi' I A = { P. domain P = I \ (\i. i \ I \ (P)\<^sub>F i \ A i) } " syntax - "_Pi'" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set" (\(3\'' _\_./ _)\ 10) + "_Pi'" :: "[pttrn, 'a set, 'b set] => ('a => 'b) set" + (\(\indent=3 notation=\binder \'\\\'' _\_./ _)\ 10) syntax_consts "_Pi'" == Pi' translations @@ -636,7 +638,8 @@ "Pi\<^sub>F I M \ PiF I M" syntax - "_PiF" :: "pttrn \ 'i set \ 'a measure \ ('i => 'a) measure" (\(3\\<^sub>F _\_./ _)\ 10) + "_PiF" :: "pttrn \ 'i set \ 'a measure \ ('i => 'a) measure" + (\(\indent=3 notation=\binder \\<^sub>F\\\\<^sub>F _\_./ _)\ 10) syntax_consts "_PiF" == PiF translations