src/HOL/MicroJava/J/TypeRel.thy
changeset 11284 981ea92a86dd
parent 11266 70c9ebbffc49
child 11372 648795477bb5
--- a/src/HOL/MicroJava/J/TypeRel.thy	Thu May 03 18:22:36 2001 +0200
+++ b/src/HOL/MicroJava/J/TypeRel.thy	Fri May 04 15:38:48 2001 +0200
@@ -74,8 +74,6 @@
 apply  auto
 done
 
-declare same_fstI [intro!] (*### TO HOL/Wellfounded_Relations *)
-
 consts class_rec ::"'c prog \<times> cname \<Rightarrow> 
         'a \<Rightarrow> (cname \<Rightarrow> fdecl list \<Rightarrow> 'c mdecl list \<Rightarrow> 'a \<Rightarrow> 'a) \<Rightarrow> 'a"
 
@@ -84,8 +82,10 @@
                          | Some (D,fs,ms) \<Rightarrow> if wf ((subcls1 G)^-1) then 
       f C fs ms (if C = Object then t else class_rec (G,D) t f) else arbitrary)"
 (hints intro: subcls1I)
+
 declare class_rec.simps [simp del]
 
+
 lemma class_rec_lemma: "\<lbrakk> wf ((subcls1 G)^-1); class G C = Some (D,fs,ms)\<rbrakk> \<Longrightarrow>
  class_rec (G,C) t f = f C fs ms (if C=Object then t else class_rec (G,D) t f)";
   apply (rule class_rec.simps [THEN trans [THEN fun_cong [THEN fun_cong]]])