src/HOL/Bali/AxCompl.thy
changeset 18459 2b102759160d
parent 18249 4398f0f12579
child 20103 26747ea32d35
equal deleted inserted replaced
18458:c0794cdbc6d1 18459:2b102759160d
  1060     fix v e c es
  1060     fix v e c es
  1061     have "G,A\<turnstile>{=:n} \<langle>v\<rangle>\<^sub>v\<succ> {G\<rightarrow>}" and 
  1061     have "G,A\<turnstile>{=:n} \<langle>v\<rangle>\<^sub>v\<succ> {G\<rightarrow>}" and 
  1062       "G,A\<turnstile>{=:n} \<langle>e\<rangle>\<^sub>e\<succ> {G\<rightarrow>}" and
  1062       "G,A\<turnstile>{=:n} \<langle>e\<rangle>\<^sub>e\<succ> {G\<rightarrow>}" and
  1063       "G,A\<turnstile>{=:n} \<langle>c\<rangle>\<^sub>s\<succ> {G\<rightarrow>}" and  
  1063       "G,A\<turnstile>{=:n} \<langle>c\<rangle>\<^sub>s\<succ> {G\<rightarrow>}" and  
  1064       "G,A\<turnstile>{=:n} \<langle>es\<rangle>\<^sub>l\<succ> {G\<rightarrow>}"
  1064       "G,A\<turnstile>{=:n} \<langle>es\<rangle>\<^sub>l\<succ> {G\<rightarrow>}"
  1065     proof (induct rule: var_expr_stmt.induct)
  1065     proof (induct rule: var_expr_stmt.inducts)
  1066       case (LVar v)
  1066       case (LVar v)
  1067       show "G,A\<turnstile>{=:n} \<langle>LVar v\<rangle>\<^sub>v\<succ> {G\<rightarrow>}"
  1067       show "G,A\<turnstile>{=:n} \<langle>LVar v\<rangle>\<^sub>v\<succ> {G\<rightarrow>}"
  1068 	apply (rule MGFn_NormalI)
  1068 	apply (rule MGFn_NormalI)
  1069 	apply (rule ax_derivs.LVar [THEN conseq1])
  1069 	apply (rule ax_derivs.LVar [THEN conseq1])
  1070 	apply (clarsimp)
  1070 	apply (clarsimp)