src/HOL/Bali/DeclConcepts.thy
changeset 13524 604d0f3622d6
parent 12962 a24ffe84a06a
child 13585 db4005b40cc6
equal deleted inserted replaced
13523:079af5c90d1c 13524:604d0f3622d6
   564                                  ("_\<turnstile> _ undeclared'_in _" [61,61,61] 60)
   564                                  ("_\<turnstile> _ undeclared'_in _" [61,61,61] 60)
   565 
   565 
   566 "G\<turnstile>m undeclared_in C \<equiv> (case m of
   566 "G\<turnstile>m undeclared_in C \<equiv> (case m of
   567                             fid fn  \<Rightarrow> cdeclaredfield G C fn  = None
   567                             fid fn  \<Rightarrow> cdeclaredfield G C fn  = None
   568                           | mid sig \<Rightarrow> cdeclaredmethd G C sig = None)"
   568                           | mid sig \<Rightarrow> cdeclaredmethd G C sig = None)"
   569 
       
   570 lemma method_declared_inI:
       
   571   "\<lbrakk>class G C = Some c; table_of (methods c) sig = Some m\<rbrakk> 
       
   572    \<Longrightarrow> G\<turnstile>mdecl (sig,m) declared_in C"
       
   573 by (auto simp add: declared_in_def cdeclaredmethd_def)
       
   574 
   569 
   575 
   570 
   576 subsubsection "members"
   571 subsubsection "members"
   577 
   572 
   578 consts
   573 consts