src/HOL/IMP/Abs_Int2_ivl.thy
changeset 55127 11408b65e9a6
parent 55125 0e0c09fca7bc
child 55565 f663fc1e653b
equal deleted inserted replaced
55126:9f9db4e6fabc 55127:11408b65e9a6
     3 theory Abs_Int2_ivl
     3 theory Abs_Int2_ivl
     4 imports Abs_Int2
     4 imports Abs_Int2
     5 begin
     5 begin
     6 
     6 
     7 subsection "Interval Analysis"
     7 subsection "Interval Analysis"
     8 
       
     9 text{* Drop @{const Fin} around numerals on output from value command: *}
       
    10 declare Fin_numeral[code_post] Fin_neg_numeral[code_post]
       
    11   zero_extended_def[symmetric, code_post] one_extended_def[symmetric, code_post]
       
    12 
     8 
    13 type_synonym eint = "int extended"
     9 type_synonym eint = "int extended"
    14 type_synonym eint2 = "eint * eint"
    10 type_synonym eint2 = "eint * eint"
    15 
    11 
    16 definition \<gamma>_rep :: "eint2 \<Rightarrow> int set" where
    12 definition \<gamma>_rep :: "eint2 \<Rightarrow> int set" where