src/HOL/IMP/Abs_Int_ITP/Abs_Int1_const_ITP.thy
changeset 55600 3c7610b8dcfc
parent 55599 6535c537b243
child 58249 180f1b3508ed
equal deleted inserted replaced
55599:6535c537b243 55600:3c7610b8dcfc
    66     by(auto simp: plus_const_cases split: const.split)
    66     by(auto simp: plus_const_cases split: const.split)
    67 qed
    67 qed
    68 
    68 
    69 permanent_interpretation Abs_Int
    69 permanent_interpretation Abs_Int
    70 where \<gamma> = \<gamma>_const and num' = Const and plus' = plus_const
    70 where \<gamma> = \<gamma>_const and num' = Const and plus' = plus_const
    71 defines AI_const is AI and step_const is step' and aval'_const is aval'
    71 defining AI_const = AI and step_const = step' and aval'_const = aval'
    72 ..
    72 ..
    73 
    73 
    74 
    74 
    75 subsubsection "Tests"
    75 subsubsection "Tests"
    76 
    76