*** empty log message ***
authornipkow
Fri, 06 Dec 2002 11:09:02 +0100
changeset 13741 ff140d072bc9
parent 13740 e3cb04713384
child 13742 452ff5d0b69d
*** empty log message ***
src/HOL/Hoare/Pointers.thy
--- a/src/HOL/Hoare/Pointers.thy	Thu Dec 05 18:44:16 2002 +0100
+++ b/src/HOL/Hoare/Pointers.thy	Fri Dec 06 11:09:02 2002 +0100
@@ -104,6 +104,13 @@
 lemma List_Ref[simp]: "List h (Ref a) as = (\<exists>bs. as = a#bs \<and> List h (h a) bs)"
 by(case_tac as, simp_all, fast)
 
+theorem notin_List_update[simp]:
+ "\<And>x. a \<notin> set as \<Longrightarrow> List (h(a := y)) x as = List h x as"
+apply(induct as)
+apply simp
+apply(clarsimp simp add:fun_upd_apply)
+done
+
 
 declare fun_upd_apply[simp del]fun_upd_same[simp] fun_upd_other[simp]
 
@@ -127,13 +134,6 @@
 apply(fastsimp dest:List_hd_not_in_tl)
 done
 
-theorem notin_List_update[simp]:
- "\<And>x. a \<notin> set as \<Longrightarrow> List (h(a := y)) x as = List h x as"
-apply(induct as)
-apply simp
-apply(clarsimp simp add:fun_upd_apply)
-done
-
 subsection "Functional abstraction"
 
 constdefs