src/HOL/ex/LocaleTest2.thy
changeset 58889 5b7a9633cfa8
parent 33657 a4179bf442d1
child 61343 5b5656a63bd6
equal deleted inserted replaced
58888:9537bf1c4853 58889:5b7a9633cfa8
     6 Definitions are less natural in FOL, since there is no selection operator.
     6 Definitions are less natural in FOL, since there is no selection operator.
     7 Hence we do them here in HOL, not in the main test suite for locales,
     7 Hence we do them here in HOL, not in the main test suite for locales,
     8 which is FOL/ex/LocaleTest.thy
     8 which is FOL/ex/LocaleTest.thy
     9 *)
     9 *)
    10 
    10 
    11 header {* Test of Locale Interpretation *}
    11 section {* Test of Locale Interpretation *}
    12 
    12 
    13 theory LocaleTest2
    13 theory LocaleTest2
    14 imports Main GCD
    14 imports Main GCD
    15 begin
    15 begin
    16 
    16