src/HOL/ex/Meson_Test.thy
changeset 32135 f645b51e8e54
parent 26732 6ea9de67e576
child 32174 9036cc8ae775
equal deleted inserted replaced
32134:ee143615019c 32135:f645b51e8e54
     1 (*ID:         $Id$*)
       
     2 
     1 
     3 header {* Meson test cases *}
     2 header {* Meson test cases *}
     4 
     3 
     5 theory Meson_Test
     4 theory Meson_Test
     6 imports Main
     5 imports Main
     9 text {*
     8 text {*
    10   WARNING: there are many potential conflicts between variables used
     9   WARNING: there are many potential conflicts between variables used
    11   below and constants declared in HOL!
    10   below and constants declared in HOL!
    12 *}
    11 *}
    13 
    12 
    14 hide const subset member quotient
    13 hide (open) const subset member quotient union inter
    15 
    14 
    16 text {*
    15 text {*
    17   Test data for the MESON proof procedure
    16   Test data for the MESON proof procedure
    18   (Excludes the equality problems 51, 52, 56, 58)
    17   (Excludes the equality problems 51, 52, 56, 58)
    19 *}
    18 *}