src/HOL/Bali/TypeSafe.thy
changeset 60751 83f04804696c
parent 58887 38db8ddc0f57
child 62042 6c6ccf573479
equal deleted inserted replaced
60750:7694aa52ad56 60751:83f04804696c
  3887                 \<rbrakk> \<Longrightarrow> P L accC (Norm s0) \<langle>If(e) c1 Else c2\<rangle>\<^sub>s \<diamondsuit> s2" 
  3887                 \<rbrakk> \<Longrightarrow> P L accC (Norm s0) \<langle>If(e) c1 Else c2\<rangle>\<^sub>s \<diamondsuit> s2" 
  3888    shows "P L accC s0 t v s1"  
  3888    shows "P L accC s0 t v s1"  
  3889 proof -
  3889 proof -
  3890   note inj_term_simps [simp]
  3890   note inj_term_simps [simp]
  3891   from eval 
  3891   from eval 
  3892   show "\<And> L accC T A. \<lbrakk>\<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>t\<Colon>T;
  3892   have "\<And>L accC T A. \<lbrakk>\<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>t\<Colon>T;
  3893                        \<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>dom (locals (store s0))\<guillemotright>t\<guillemotright>A\<rbrakk>  
  3893                        \<lparr>prg=G,cls=accC,lcl=L\<rparr>\<turnstile>dom (locals (store s0))\<guillemotright>t\<guillemotright>A\<rbrakk>  
  3894         \<Longrightarrow> P L accC s0 t v s1" (is "PROP ?Hyp s0 t v s1")
  3894         \<Longrightarrow> P L accC s0 t v s1" (is "PROP ?Hyp s0 t v s1")
  3895   proof (induct)
  3895   proof (induct)
  3896     case Abrupt with abrupt show ?case .
  3896     case Abrupt with abrupt show ?case .
  3897   next
  3897   next