src/HOL/ex/BinEx.thy
changeset 16417 9bc16273c2d4
parent 15965 f422f8283491
child 20807 bd3b60f9a343
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4     Copyright   1998  University of Cambridge
     4     Copyright   1998  University of Cambridge
     5 *)
     5 *)
     6 
     6 
     7 header {* Binary arithmetic examples *}
     7 header {* Binary arithmetic examples *}
     8 
     8 
     9 theory BinEx = Main:
     9 theory BinEx imports Main begin
    10 
    10 
    11 subsection {* Regression Testing for Cancellation Simprocs *}
    11 subsection {* Regression Testing for Cancellation Simprocs *}
    12 
    12 
    13 (*taken from HOL/Integ/int_arith1.ML *)
    13 (*taken from HOL/Integ/int_arith1.ML *)
    14 
    14