src/HOL/IMP/Abs_Int_ITP/Abs_Int2_ivl_ITP.thy
changeset 48480 cb03acfae211
parent 47602 3d44790b5ab0
child 55599 6535c537b243
equal deleted inserted replaced
48479:819f7a5f3e7f 48480:cb03acfae211
     1 (* Author: Tobias Nipkow *)
     1 (* Author: Tobias Nipkow *)
     2 
     2 
     3 theory Abs_Int2_ivl_ITP
     3 theory Abs_Int2_ivl_ITP
     4 imports Abs_Int2_ITP Abs_Int_Tests
     4 imports Abs_Int2_ITP "../Abs_Int_Tests"
     5 begin
     5 begin
     6 
     6 
     7 subsection "Interval Analysis"
     7 subsection "Interval Analysis"
     8 
     8 
     9 datatype ivl = I "int option" "int option"
     9 datatype ivl = I "int option" "int option"