diff -r 9171d1ce5a35 -r 53982d5ec0bb src/ZF/UNITY/UNITY.thy --- a/src/ZF/UNITY/UNITY.thy Thu Jan 03 21:06:39 2019 +0100 +++ b/src/ZF/UNITY/UNITY.thy Thu Jan 03 21:15:52 2019 +0100 @@ -27,7 +27,7 @@ cons(id(state), allowed \ Pow(state*state))>" definition - SKIP :: i ("\") where + SKIP :: i (\\\) where "SKIP == mk_program(state, 0, Pow(state*state))" (* Coercion from anything to program *) @@ -68,12 +68,12 @@ initially :: "i=>i" where "initially(A) == {F \ program. Init(F)\A}" -definition "constrains" :: "[i, i] => i" (infixl "co" 60) where +definition "constrains" :: "[i, i] => i" (infixl \co\ 60) where "A co B == {F \ program. (\act \ Acts(F). act``A\B) & st_set(A)}" \ \the condition @{term "st_set(A)"} makes the definition slightly stronger than the HOL one\ -definition unless :: "[i, i] => i" (infixl "unless" 60) where +definition unless :: "[i, i] => i" (infixl \unless\ 60) where "A unless B == (A - B) co (A \ B)" definition @@ -90,7 +90,7 @@ (* meta-function composition *) definition - metacomp :: "[i=>i, i=>i] => (i=>i)" (infixl "comp" 65) where + metacomp :: "[i=>i, i=>i] => (i=>i)" (infixl \comp\ 65) where "f comp g == %x. f(g(x))" definition