fix for change in nat number simplification
authorkleing
Sat, 11 May 2002 20:40:31 +0200
changeset 13139 94648e0e4506
parent 13138 6568fee2bd3a
child 13140 6d97dbb189a9
fix for change in nat number simplification
src/HOL/MicroJava/BV/BVExample.thy
--- a/src/HOL/MicroJava/BV/BVExample.thy	Sat May 11 20:27:13 2002 +0200
+++ b/src/HOL/MicroJava/BV/BVExample.thy	Sat May 11 20:40:31 2002 +0200
@@ -253,6 +253,8 @@
    (                                    [], [Class list_name, Class list_name]),
    (                          [PrimT Void], [Class list_name, Class list_name])]"
 
+declare nat_number [simp]
+
 lemma wt_append [simp]:
   "wt_method E list_name [Class list_name] (PrimT Void) 3 0 append_ins
              [(Suc 0, 2, 8, Xcpt NullPointer)] \<phi>\<^sub>a"
@@ -348,7 +350,9 @@
   Phi :: prog_type ("\<Phi>")
   "\<Phi> C sg \<equiv> if C = test_name \<and> sg = (makelist_name, []) then \<phi>\<^sub>m else          
              if C = list_name \<and> sg = (append_name, [Class list_name]) then \<phi>\<^sub>a else []"
-  
+
+declare nat_number [simp del]   
+
 lemma wf_prog:
   "wt_jvm_prog E \<Phi>" 
   apply (unfold wt_jvm_prog_def)