diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/UNITY/Constrains.thy --- a/src/HOL/UNITY/Constrains.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/UNITY/Constrains.thy Fri Sep 20 19:51:08 2024 +0200 @@ -32,10 +32,10 @@ | Acts: "[| act \ Acts F; s \ reachable F; (s,s') \ act |] ==> s' \ reachable F" -definition Constrains :: "['a set, 'a set] => 'a program set" (infixl "Co" 60) where +definition Constrains :: "['a set, 'a set] => 'a program set" (infixl \Co\ 60) where "A Co B == {F. F \ (reachable F \ A) co B}" -definition Unless :: "['a set, 'a set] => 'a program set" (infixl "Unless" 60) where +definition Unless :: "['a set, 'a set] => 'a program set" (infixl \Unless\ 60) where "A Unless B == (A-B) Co (A \ B)" definition Stable :: "'a set => 'a program set" where