src/HOL/MicroJava/J/JListExample.thy
changeset 45827 66c68453455c
parent 45231 d85a2fdc586c
child 46506 c7faa011bfa7
--- a/src/HOL/MicroJava/J/JListExample.thy	Tue Dec 13 14:04:20 2011 +0100
+++ b/src/HOL/MicroJava/J/JListExample.thy	Tue Dec 13 15:18:52 2011 +0100
@@ -111,7 +111,9 @@
   "HOL.equal l4_nam l3_nam \<longleftrightarrow> False"
   by(simp_all add: distinct_fields distinct_fields[symmetric] distinct_vars distinct_vars[symmetric] equal_vnam_def)
 
-axioms nat_to_loc'_inject: "nat_to_loc' l = nat_to_loc' l' \<longleftrightarrow> l = l'"
+axiomatization where
+  nat_to_loc'_inject: "nat_to_loc' l = nat_to_loc' l' \<longleftrightarrow> l = l'"
+
 lemma equal_loc'_code [code]:
   "HOL.equal (nat_to_loc' l) (nat_to_loc' l') \<longleftrightarrow> l = l'"
   by(simp add: equal_loc'_def nat_to_loc'_inject)