src/HOL/TLA/Memory/RPCParameters.thy
changeset 60587 0318b43ee95c
parent 58889 5b7a9633cfa8
child 60588 750c533459b1
--- a/src/HOL/TLA/Memory/RPCParameters.thy	Fri Jun 26 11:07:04 2015 +0200
+++ b/src/HOL/TLA/Memory/RPCParameters.thy	Fri Jun 26 11:44:22 2015 +0200
@@ -30,10 +30,10 @@
 
 axiomatization where
   (* RPCFailure is different from MemVals and exceptions *)
-  RFNoMemVal:        "RPCFailure ~: MemVal" and
-  NotAResultNotRF:   "NotAResult ~= RPCFailure" and
-  OKNotRF:           "OK ~= RPCFailure" and
-  BANotRF:           "BadArg ~= RPCFailure"
+  RFNoMemVal:        "RPCFailure \<notin> MemVal" and
+  NotAResultNotRF:   "NotAResult \<noteq> RPCFailure" and
+  OKNotRF:           "OK \<noteq> RPCFailure" and
+  BANotRF:           "BadArg \<noteq> RPCFailure"
 
 defs
   IsLegalRcvArg_def: "IsLegalRcvArg ra ==