slight cleanup
authorhaftmann
Fri, 20 Oct 2006 10:44:42 +0200
changeset 21063 3c5074f028c8
parent 21062 876dd2695423
child 21064 9684dd7c81b5
slight cleanup
src/HOL/Library/ExecutableSet.thy
src/HOL/MicroJava/JVM/JVMListExample.thy
--- a/src/HOL/Library/ExecutableSet.thy	Fri Oct 20 10:44:39 2006 +0200
+++ b/src/HOL/Library/ExecutableSet.thy	Fri Oct 20 10:44:42 2006 +0200
@@ -13,7 +13,7 @@
 
 instance set :: (eq) eq ..
 
-lemma [code target: Set]:
+lemma [code target: Set, code nofunc]:
   "(A = B) = (A \<subseteq> B \<and> B \<subseteq> A)"
   by blast
 
@@ -240,11 +240,9 @@
   "ExecutableSet.insertl" "List.insertl"
   "ExecutableSet.drop_first" "List.drop_first"
 
-definition
+definition [code inline]:
   "empty_list = []"
 
-declare empty_list_def [code inline]
-
 lemma [code func]:
   "insert (x \<Colon> 'a\<Colon>eq) = insert x" ..
 
--- a/src/HOL/MicroJava/JVM/JVMListExample.thy	Fri Oct 20 10:44:39 2006 +0200
+++ b/src/HOL/MicroJava/JVM/JVMListExample.thy	Fri Oct 20 10:44:42 2006 +0200
@@ -120,22 +120,20 @@
   and vname :: eq
   and mname :: eq
   and ty :: eq
+  and val :: eq
   and instr :: eq ..
 
 definition
   arbitrary_val :: val
-  "arbitrary_val = arbitrary"
+  [symmetric, code inline]: "arbitrary_val = arbitrary"
   arbitrary_cname :: cname
-  "arbitrary_cname = arbitrary"
-
-declare arbitrary_val_def [symmetric, code inline]
-declare arbitrary_cname_def [symmetric, code inline]
+  [symmetric, code inline]: "arbitrary_cname = arbitrary"
 
 definition
   "unit' = Unit"
   "object' = Object"
 
-code_constsubst
+code_axioms
   arbitrary_val \<equiv> unit'
   arbitrary_cname \<equiv> object'
 
@@ -165,7 +163,7 @@
 code_const
   wf_class (SML target_atom "(fn _ => true)")
 
-code_constsubst
+code_axioms
   new_Addr \<equiv> new_addr'
 
 definition