diff -r 5eb932e604a2 -r eab6ce8368fa src/HOL/IMP/Abs_Int3.thy --- a/src/HOL/IMP/Abs_Int3.thy Wed Jan 10 15:21:49 2018 +0100 +++ b/src/HOL/IMP/Abs_Int3.thy Wed Jan 10 15:25:09 2018 +0100 @@ -56,10 +56,10 @@ instantiation st :: ("{order_top,wn}")wn begin -lift_definition widen_st :: "'a st \ 'a st \ 'a st" is "map2_st_rep (op \)" +lift_definition widen_st :: "'a st \ 'a st \ 'a st" is "map2_st_rep (\)" by(auto simp: eq_st_def) -lift_definition narrow_st :: "'a st \ 'a st \ 'a st" is "map2_st_rep (op \)" +lift_definition narrow_st :: "'a st \ 'a st \ 'a st" is "map2_st_rep (\)" by(auto simp: eq_st_def) instance @@ -113,13 +113,13 @@ instantiation acom :: (widen)widen begin -definition "widen_acom = map2_acom (op \)" +definition "widen_acom = map2_acom (\)" instance .. end instantiation acom :: (narrow)narrow begin -definition "narrow_acom = map2_acom (op \)" +definition "narrow_acom = map2_acom (\)" instance .. end @@ -255,7 +255,7 @@ end global_interpretation Abs_Int_wn -where \ = \_ivl and num' = num_ivl and plus' = "op +" +where \ = \_ivl and num' = num_ivl and plus' = "(+)" and test_num' = in_ivl and inv_plus' = inv_plus_ivl and inv_less' = inv_less_ivl defines AI_wn_ivl = AI_wn @@ -540,7 +540,7 @@ global_interpretation Abs_Int_wn_measure -where \ = \_ivl and num' = num_ivl and plus' = "op +" +where \ = \_ivl and num' = num_ivl and plus' = "(+)" and test_num' = in_ivl and inv_plus' = inv_plus_ivl and inv_less' = inv_less_ivl and m = m_ivl and n = n_ivl and h = 3