src/HOL/MicroJava/BV/JVMType.thy
changeset 13672 b95d12325b51
parent 13006 51c5f3f11d16
child 14025 d9b155757dc8
equal deleted inserted replaced
13671:eec2582923f6 13672:b95d12325b51
   209   by (simp add: sup_loc_def Listn.le_def lesub_def list_all2_Cons1)
   209   by (simp add: sup_loc_def Listn.le_def lesub_def list_all2_Cons1)
   210 
   210 
   211 theorem sup_loc_Cons2:
   211 theorem sup_loc_Cons2:
   212   "(G \<turnstile> YT <=l (X#XT)) = (\<exists>Y YT'. YT=Y#YT' \<and> (G \<turnstile> Y <=o X) \<and> (G \<turnstile> YT' <=l XT))"
   212   "(G \<turnstile> YT <=l (X#XT)) = (\<exists>Y YT'. YT=Y#YT' \<and> (G \<turnstile> Y <=o X) \<and> (G \<turnstile> YT' <=l XT))"
   213   by (simp add: sup_loc_def Listn.le_def lesub_def list_all2_Cons2)
   213   by (simp add: sup_loc_def Listn.le_def lesub_def list_all2_Cons2)
       
   214 
       
   215 lemma sup_state_Cons:
       
   216   "(G \<turnstile> (x#xt, a) <=s (y#yt, b)) = 
       
   217    ((G \<turnstile> x \<preceq> y) \<and> (G \<turnstile> (xt,a) <=s (yt,b)))"
       
   218   by (auto simp add: sup_state_def stk_convert lesub_def Product.le_def)
   214 
   219 
   215 
   220 
   216 theorem sup_loc_length:
   221 theorem sup_loc_length:
   217   "G \<turnstile> a <=l b \<Longrightarrow> length a = length b"
   222   "G \<turnstile> a <=l b \<Longrightarrow> length a = length b"
   218 proof -
   223 proof -