src/HOL/IMP/Abs_State.thy
changeset 45127 d2eb07a1e01b
parent 45111 054a9ac0d7ef
child 45212 e87feee00a4c
--- a/src/HOL/IMP/Abs_State.thy	Mon Oct 10 20:14:25 2011 +0200
+++ b/src/HOL/IMP/Abs_State.thy	Wed Oct 12 09:16:30 2011 +0200
@@ -24,6 +24,7 @@
 "show_st_up (Up S) = Up(show_st S)"
 
 definition "show_acom = map_acom show_st_up"
+definition "show_acom_opt = Option.map show_acom"
 
 definition "lookup F x = (if x : set(dom F) then fun F x else \<top>)"
 
@@ -61,10 +62,10 @@
 lemma mono_update: "a \<sqsubseteq> a' \<Longrightarrow> S \<sqsubseteq> S' \<Longrightarrow> update S x a \<sqsubseteq> update S' x a'"
 by(auto simp add: le_st_def lookup_def update_def)
 
-context Rep
+context Val_abs
 begin
 
-abbreviation fun_in_rep :: "(name \<Rightarrow> 'b) \<Rightarrow> 'a st \<Rightarrow> bool" (infix "<:f" 50) where
+abbreviation fun_in_rep :: "state \<Rightarrow> 'a st \<Rightarrow> bool" (infix "<:f" 50) where
 "s <:f S == s \<in> rep_st rep S"
 
 notation fun_in_rep (infix "<:\<^sub>f" 50)
@@ -73,7 +74,7 @@
 apply(auto simp add: rep_st_def le_st_def dest: le_rep)
 by (metis in_rep_Top le_rep lookup_def subsetD)
 
-abbreviation in_rep_up :: "(name \<Rightarrow> 'b) \<Rightarrow> 'a st up \<Rightarrow> bool"  (infix "<:up" 50)
+abbreviation in_rep_up :: "state \<Rightarrow> 'a st up \<Rightarrow> bool"  (infix "<:up" 50)
 where "s <:up S == s : rep_up (rep_st rep) S"
 
 notation (output) in_rep_up (infix "<:\<^sub>u\<^sub>p" 50)