src/HOL/IMP/Abs_Int_ITP/Abs_Int3_ITP.thy
changeset 61890 f6ded81f5690
parent 61671 20d4cd2ceab2
child 62378 85ed00c1fe7c
equal deleted inserted replaced
61857:542f2c6da692 61890:f6ded81f5690
   223     by (blast intro: mono_gamma_c order_trans)
   223     by (blast intro: mono_gamma_c order_trans)
   224 qed
   224 qed
   225 
   225 
   226 end
   226 end
   227 
   227 
   228 permanent_interpretation Abs_Int2
   228 global_interpretation Abs_Int2
   229 where \<gamma> = \<gamma>_ivl and num' = num_ivl and plus' = plus_ivl
   229 where \<gamma> = \<gamma>_ivl and num' = num_ivl and plus' = plus_ivl
   230 and test_num' = in_ivl
   230 and test_num' = in_ivl
   231 and filter_plus' = filter_plus_ivl and filter_less' = filter_less_ivl
   231 and filter_plus' = filter_plus_ivl and filter_less' = filter_less_ivl
   232 defines AI_ivl' = AI_wn
   232 defines AI_ivl' = AI_wn
   233 ..
   233 ..