test/Tools/isac/ADDTESTS/file-depend/Build_Test.thy
author Walther Neuper <neuper@ist.tugraz.at>
Tue, 31 Aug 2010 15:36:57 +0200
branchisac-update-Isa09-2
changeset 37965 9c11005c33b8
parent 37949 aaf528d3ebd5
child 41899 d837e83a4835
permissions -rw-r--r--
updated Knowledge/Atools.thy + some changes + changes ahead

# replaced thms ahead by ./thms-replace-Isa02-Isa09-2.sml
# Knowledge/Delete.thy takes intermediate code:
* fun calc, fun term_of_float,fun var_op_float, fun float_op_var
for Float, which have already been deleted
* thms which are available only with long.identifiers
which cannot be handled in isac's Scripts
# added ProgLang/Language.thy collecting all data about Scripts
     1 (*
     2 $ cd /usr/local/isabisac/test/Tools/isac/ADDTESTS/file-depend
     3 $ /usr/local/isabisac/bin/isabelle emacs Build_Test.thy &
     4 
     5 *)
     6 
     7 theory Build_Test imports Complex_Main begin
     8 
     9 use     "0foolibrary.ML"
    10 use_thy "1language/Foo_Language"
    11 use     "2interpreter/2foointerpreter.ML"
    12 
    13 (*vvvvvvv can be bypassed with Foo_KnowALL
    14 use_thy "3knowledge/Foo_Know111"
    15 use_thy "3knowledge/Foo_Know222"
    16   ^^^^^^^ can be bypassed with Foo_KnowALL*)
    17 use_thy "3knowledge/Foo_KnowALL"
    18 
    19 text {* the different theories of knowledge are recognized, Const bar*: *}
    20 ML {* 
    21 val trm = Syntax.read_term_global @{theory Foo_Know111} 
    22   "fooprog (foo111 = bar111)";
    23 val Const ("Foo_Know111.bar111", _) = foointerpret trm;
    24 
    25 val trm = Syntax.read_term_global @{theory Foo_Know222} 
    26   "fooprog (foo222 = bar222)";
    27 val Const ("Foo_Know222.bar222", _) = foointerpret trm;
    28 *}
    29 
    30 text {* the different theories of knowledge are recognized, Free bar*: *}
    31 ML {*
    32 val trm = Syntax.read_term_global @{theory Foo_Know111} 
    33   "fooprog (foo222 = bar222)";
    34 (*Const ("Foo_Language.fooprog", "bool => Foo_Language.foosource") $
    35      (Const ("op =", "'a => 'a => bool") $ Free ("foo222", "'a") $
    36        Free ("bar222", "'a"))
    37    : term*)
    38 
    39 val trm = Syntax.read_term_global @{theory Foo_Know222} 
    40   "fooprog (foo111 = bar111)";
    41 (*val trm =
    42    Const ("Foo_Language.fooprog", "bool => Foo_Language.foosource") $
    43      (Const ("op =", "'a => 'a => bool") $ Free ("foo111", "'a") $
    44        Free ("bar111", "'a"))
    45    : term*)
    46 *}