src/HOL/IMP/Abs_State.thy
changeset 52504 52cd8bebc3b6
parent 52020 db08e493cf44
child 52729 412c9e0381a1
--- a/src/HOL/IMP/Abs_State.thy	Tue Jul 02 20:47:32 2013 +0200
+++ b/src/HOL/IMP/Abs_State.thy	Wed Jul 03 16:07:00 2013 +0200
@@ -128,7 +128,7 @@
 lemma mono_fun: "S1 \<le> S2 \<Longrightarrow> fun S1 x \<le> fun S2 x"
 by transfer (simp add: less_eq_st_rep_iff)
 
-locale Gamma = Val_abs where \<gamma>=\<gamma>
+locale Gamma_semilattice = Val_semilattice where \<gamma>=\<gamma>
   for \<gamma> :: "'av::semilattice_sup_top \<Rightarrow> val set"
 begin