src/HOL/MicroJava/BV/Correct.thy
changeset 59199 cb8e5f7a5e4a
parent 58886 8a6cac7c7247
child 60773 d09c66a0ea10
equal deleted inserted replaced
59198:c73933e07c03 59199:cb8e5f7a5e4a
   173 subsection {* approx-stk *}
   173 subsection {* approx-stk *}
   174 
   174 
   175 lemma approx_stk_rev_lem:
   175 lemma approx_stk_rev_lem:
   176   "approx_stk G hp (rev s) (rev t) = approx_stk G hp s t"
   176   "approx_stk G hp (rev s) (rev t) = approx_stk G hp s t"
   177   apply (unfold approx_stk_def approx_loc_def)
   177   apply (unfold approx_stk_def approx_loc_def)
   178   apply (simp add: rev_map [THEN sym])
   178   apply (simp add: rev_map [symmetric])
   179   done
   179   done
   180 
   180 
   181 lemma approx_stk_rev:
   181 lemma approx_stk_rev:
   182   "approx_stk G hp (rev s) t = approx_stk G hp s (rev t)"
   182   "approx_stk G hp (rev s) t = approx_stk G hp s (rev t)"
   183   by (auto intro: subst [OF approx_stk_rev_lem])
   183   by (auto intro: subst [OF approx_stk_rev_lem])