src/HOL/TLA/Memory/MemoryParameters.thy
changeset 47968 3119ad2b5ad3
parent 41589 bbd861837ebc
child 58249 180f1b3508ed
--- a/src/HOL/TLA/Memory/MemoryParameters.thy	Wed May 23 16:22:27 2012 +0200
+++ b/src/HOL/TLA/Memory/MemoryParameters.thy	Wed May 23 16:53:12 2012 +0200
@@ -25,14 +25,14 @@
   (* the initial value stored in each memory cell *)
   InitVal        :: "Vals"
 
-axioms
+axiomatization where
   (* basic assumptions about the above constants and predicates *)
-  BadArgNoMemVal:    "BadArg ~: MemVal"
-  MemFailNoMemVal:   "MemFailure ~: MemVal"
-  InitValMemVal:     "InitVal : MemVal"
-  NotAResultNotVal:  "NotAResult ~: MemVal"
-  NotAResultNotOK:   "NotAResult ~= OK"
-  NotAResultNotBA:   "NotAResult ~= BadArg"
+  BadArgNoMemVal:    "BadArg ~: MemVal" and
+  MemFailNoMemVal:   "MemFailure ~: MemVal" and
+  InitValMemVal:     "InitVal : MemVal" and
+  NotAResultNotVal:  "NotAResult ~: MemVal" and
+  NotAResultNotOK:   "NotAResult ~= OK" and
+  NotAResultNotBA:   "NotAResult ~= BadArg" and
   NotAResultNotMF:   "NotAResult ~= MemFailure"
 
 lemmas [simp] =