changeset 67445 | 4311845b0412 |
parent 67443 | 3abf6a722518 |
child 76213 | e44d86131648 |
--- a/src/ZF/UNITY/Mutex.thy Tue Jan 16 09:58:06 2018 +0100 +++ b/src/ZF/UNITY/Mutex.thy Tue Jan 16 09:58:17 2018 +0100 @@ -27,7 +27,7 @@ abbreviation "u == Var([0,1])" abbreviation "v == Var([1,0])" -axiomatization where \<comment> \<open>* Type declarations *\<close> +axiomatization where \<comment> \<open>Type declarations\<close> 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