src/HOL/MicroJava/Comp/Index.thy
changeset 14045 a34d89ce6097
parent 13737 e564c3d2d174
child 14981 e73f8140af78
--- a/src/HOL/MicroJava/Comp/Index.thy	Mon May 26 11:42:41 2003 +0200
+++ b/src/HOL/MicroJava/Comp/Index.thy	Mon May 26 18:36:15 2003 +0200
@@ -63,6 +63,10 @@
 apply simp
 done
 
+lemma lift_if: "(f (if b then t else e)) = (if b then (f t) else (f e))"
+apply auto
+done
+
 lemma update_at_index: "
   \<lbrakk> distinct (gjmb_plns (gmb G C S)); 
   x \<in> set (gjmb_plns (gmb G C S)); x \<noteq> This \<rbrakk> \<Longrightarrow>