tuned
authornipkow
Fri, 10 May 2013 06:34:29 +0200
changeset 51926 25ceb5fa8f78
parent 51925 e3b7917186f1
child 51927 bcd6898ac613
tuned
src/HOL/IMP/Abs_Int1.thy
--- a/src/HOL/IMP/Abs_Int1.thy	Thu May 09 20:44:37 2013 +0200
+++ b/src/HOL/IMP/Abs_Int1.thy	Fri May 10 06:34:29 2013 +0200
@@ -134,14 +134,14 @@
 
 end
 
-fun top_on_st :: "'a::top st \<Rightarrow> vname set \<Rightarrow> bool" where
+fun top_on_st :: "'a::top st \<Rightarrow> vname set \<Rightarrow> bool" ("top'_on\<^isub>s") where
 "top_on_st S X = (\<forall>x\<in>X. fun S x = \<top>)"
 
-fun top_on_opt :: "'a::top st option \<Rightarrow> vname set \<Rightarrow> bool" where
+fun top_on_opt :: "'a::top st option \<Rightarrow> vname set \<Rightarrow> bool" ("top'_on\<^isub>o") where
 "top_on_opt (Some S)  X = top_on_st S X" |
 "top_on_opt None X = True"
 
-definition top_on_acom :: "'a::top st option acom \<Rightarrow> vname set \<Rightarrow> bool" where
+definition top_on_acom :: "'a::top st option acom \<Rightarrow> vname set \<Rightarrow> bool" ("top'_on\<^isub>c") where
 "top_on_acom C X = (\<forall>a \<in> set(annos C). top_on_opt a X)"
 
 lemma top_on_top: "top_on_opt (\<top>::_ st option) X"