src/HOL/ex/Simproc_Tests.thy
changeset 58889 5b7a9633cfa8
parent 51717 9e7d1c139569
child 59867 58043346ca64
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     1 (*  Title:      HOL/ex/Simproc_Tests.thy
     1 (*  Title:      HOL/ex/Simproc_Tests.thy
     2     Author:     Brian Huffman
     2     Author:     Brian Huffman
     3 *)
     3 *)
     4 
     4 
     5 header {* Testing of arithmetic simprocs *}
     5 section {* Testing of arithmetic simprocs *}
     6 
     6 
     7 theory Simproc_Tests
     7 theory Simproc_Tests
     8 imports Main
     8 imports Main
     9 begin
     9 begin
    10 
    10