src/HOL/IMP/Abs_Int1_const.thy
changeset 58249 180f1b3508ed
parent 55600 3c7610b8dcfc
child 58310 91ea607a34d8
equal deleted inserted replaced
58248:25af24e1f37b 58249:180f1b3508ed
     4 imports Abs_Int1
     4 imports Abs_Int1
     5 begin
     5 begin
     6 
     6 
     7 subsection "Constant Propagation"
     7 subsection "Constant Propagation"
     8 
     8 
     9 datatype const = Const val | Any
     9 datatype_new const = Const val | Any
    10 
    10 
    11 fun \<gamma>_const where
    11 fun \<gamma>_const where
    12 "\<gamma>_const (Const i) = {i}" |
    12 "\<gamma>_const (Const i) = {i}" |
    13 "\<gamma>_const (Any) = UNIV"
    13 "\<gamma>_const (Any) = UNIV"
    14 
    14