diff -r f075640b8868 -r 3abf6a722518 src/ZF/UNITY/Mutex.thy --- a/src/ZF/UNITY/Mutex.thy Tue Jan 16 09:12:16 2018 +0100 +++ b/src/ZF/UNITY/Mutex.thy Tue Jan 16 09:30:00 2018 +0100 @@ -27,7 +27,7 @@ abbreviation "u == Var([0,1])" abbreviation "v == Var([1,0])" -axiomatization where \\* Type declarations *\ +axiomatization where \ \* Type declarations *\ p_type: "type_of(p)=bool & default_val(p)=0" and m_type: "type_of(m)=int & default_val(m)=#0" and n_type: "type_of(n)=int & default_val(n)=#0" and