diff -r 750b63fa4c4e -r 52cd8bebc3b6 src/HOL/IMP/Abs_Int2.thy --- a/src/HOL/IMP/Abs_Int2.thy Tue Jul 02 20:47:32 2013 +0200 +++ b/src/HOL/IMP/Abs_Int2.thy Wed Jul 03 16:07:00 2013 +0200 @@ -28,7 +28,7 @@ subclass (in bounded_lattice) semilattice_sup_top .. -locale Val_abs1_gamma = Gamma where \ = \ +locale Val_lattice_gamma = Gamma_semilattice where \ = \ for \ :: "'av::bounded_lattice \ val set" + assumes inter_gamma_subset_gamma_inf: "\ a1 \ \ a2 \ \(a1 \ a2)" @@ -45,7 +45,7 @@ end -locale Val_abs1 = Val_abs1_gamma where \ = \ +locale Val_inv = Val_lattice_gamma where \ = \ for \ :: "'av::bounded_lattice \ val set" + fixes test_num' :: "val \ 'av \ bool" and inv_plus' :: "'av \ 'av \ 'av \ 'av * 'av" @@ -57,7 +57,7 @@ i1 : \ a1 \ i2 : \ a2 \ i1 : \ a\<^isub>1' \ i2 : \ a\<^isub>2'" -locale Abs_Int1 = Val_abs1 where \ = \ +locale Abs_Int_inv = Val_inv where \ = \ for \ :: "'av::bounded_lattice \ val set" begin @@ -184,7 +184,7 @@ subsubsection "Monotonicity" -locale Abs_Int1_mono = Abs_Int1 + +locale Abs_Int_inv_mono = Abs_Int_inv + assumes mono_plus': "a1 \ b1 \ a2 \ b2 \ plus' a1 a2 \ plus' b1 b2" and mono_inv_plus': "a1 \ b1 \ a2 \ b2 \ r \ r' \ inv_plus' r a1 a2 \ inv_plus' r' b1 b2"