diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/HOLCF/IOA/Automata.thy --- a/src/HOL/HOLCF/IOA/Automata.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/HOLCF/IOA/Automata.thy Fri Sep 20 19:51:08 2024 +0200 @@ -26,7 +26,7 @@ definition trans_of :: "('a, 's) ioa \ ('a, 's) transition set" where "trans_of = fst \ snd \ snd" -abbreviation trans_of_syn ("_ \_\_\ _" [81, 81, 81, 81] 100) +abbreviation trans_of_syn (\_ \_\_\ _\ [81, 81, 81, 81] 100) where "s \a\A\ t \ (s, a, t) \ trans_of A" definition wfair_of :: "('a, 's) ioa \ 'a set set" @@ -91,7 +91,7 @@ (outputs a1 \ outputs a2), (internals a1 \ internals a2)))" -definition par :: "('a, 's) ioa \ ('a, 't) ioa \ ('a, 's * 't) ioa" (infixr "\" 10) +definition par :: "('a, 's) ioa \ ('a, 't) ioa \ ('a, 's * 't) ioa" (infixr \\\ 10) where "(A \ B) = (asig_comp (asig_of A) (asig_of B), {pr. fst pr \ starts_of A \ snd pr \ starts_of B},