diff -r 3e3e7a68cd80 -r 6ad2c917dd2e src/HOL/Algebra/Coset.thy --- a/src/HOL/Algebra/Coset.thy Wed Oct 09 22:01:33 2024 +0200 +++ b/src/HOL/Algebra/Coset.thy Wed Oct 09 23:38:29 2024 +0200 @@ -19,7 +19,8 @@ where "a <#\<^bsub>G\<^esub> H = (\h\H. {a \\<^bsub>G\<^esub> h})" definition - RCOSETS :: "[_, 'a set] \ ('a set)set" (\rcosets\ _\ [81] 80) + RCOSETS :: "[_, 'a set] \ ('a set)set" + (\(\open_block notation=\prefix rcosets\\rcosets\ _)\ [81] 80) where "rcosets\<^bsub>G\<^esub> H = (\a\carrier G. {H #>\<^bsub>G\<^esub> a})" definition @@ -27,7 +28,8 @@ where "H <#>\<^bsub>G\<^esub> K = (\h\H. \k\K. {h \\<^bsub>G\<^esub> k})" definition - SET_INV :: "[_,'a set] \ 'a set" (\set'_inv\ _\ [81] 80) + SET_INV :: "[_,'a set] \ 'a set" + (\(\open_block notation=\prefix set_inv\\set'_inv\ _)\ [81] 80) where "set_inv\<^bsub>G\<^esub> H = (\h\H. {inv\<^bsub>G\<^esub> h})" @@ -659,7 +661,8 @@ subsubsection\An Equivalence Relation\ definition - r_congruent :: "[('a,'b)monoid_scheme, 'a set] \ ('a*'a)set" (\rcong\ _\) + r_congruent :: "[('a,'b)monoid_scheme, 'a set] \ ('a*'a)set" + (\(\open_block notation=\prefix rcong\\rcong\ _)\) where "rcong\<^bsub>G\<^esub> H = {(x,y). x \ carrier G \ y \ carrier G \ inv\<^bsub>G\<^esub> x \\<^bsub>G\<^esub> y \ H}"