src/Tools/isac/Build_Isac.thy
author Walther Neuper <neuper@ist.tugraz.at>
Fri, 04 May 2012 08:51:42 +0200
changeset 42412 52cb88544681
parent 42407 81afb8eb9b03
child 48760 5e1e45b3ddef
permissions -rw-r--r--
made 3 exps SignalProcessing run

Inverse_Z_Transform.thy now contains an exact cp from Build_Inver...thy
TODOL reformat
neuper@38070
     1
(*  Title:  build and test isac 
neuper@38057
     2
    Author: Walther Neuper, TU Graz, 100808
neuper@38051
     3
   (c) due to copyright terms
neuper@38051
     4
neuper@38057
     5
create a new Isac heap (via ~~/ROOT.ML) with
neuper@38057
     6
$ /usr/local/isabisac/bin/isabelle usedir -b HOL Isac
neuper@38057
     7
neuper@42400
     8
start with heap Isac
neuper@38063
     9
$ /usr/local/isabisac/bin/isabelle jedit -l Isac Build_Isac.thy &
neuper@38063
    10
neuper@37924
    11
12345678901234567890123456789012345678901234567890123456789012345678901234567890
neuper@37924
    12
        10        20        30        40        50        60        70        80
neuper@37906
    13
*)
neuper@37906
    14
neuper@37906
    15
header {* Loading the isac mathengine *}
neuper@37906
    16
neuper@41905
    17
theory Build_Isac imports Complex_Main
neuper@41905
    18
(* use    "library.sml"
neuper@41905
    19
   use    "calcelems.sml"
neuper@41905
    20
neuper@41905
    21
   use    "ProgLang/termC.sml"
neuper@41905
    22
   use    "ProgLang/calculate.sml"
neuper@41905
    23
   use    "ProgLang/rewrite.sml"
neuper@41905
    24
  "use_thy ProgLang/ListC"
neuper@41905
    25
  "use_thy ProgLang/Tools"
neuper@41905
    26
  "use_thy ProgLang/Script"
neuper@41905
    27
   use    "ProgLang/scrtools.sml"
neuper@41943
    28
*)        "ProgLang/ProgLang"
neuper@41905
    29
neuper@41905
    30
(* use    "Interpret/mstools.sml"
neuper@41905
    31
   use    "Interpret/ctree.sml"
neuper@41905
    32
   use    "Interpret/ptyps.sml"
neuper@41905
    33
   use    "Interpret/generate.sml"
neuper@41905
    34
   use    "Interpret/calchead.sml"
neuper@41905
    35
   use    "Interpret/appl.sml"
neuper@41905
    36
   use    "Interpret/rewtools.sml"
neuper@41905
    37
   use    "Interpret/script.sml"
neuper@41905
    38
   use    "Interpret/solve.sml"
neuper@41905
    39
   use    "Interpret/inform.sml"
neuper@41905
    40
   use    "Interpret/mathengine.sml"
neuper@41905
    41
*)        "Interpret/Interpret"
neuper@41905
    42
neuper@41905
    43
(* use    "xmlsrc/mathml.sml"
neuper@41905
    44
   use    "xmlsrc/datatypes.sml"
neuper@41905
    45
   use    "xmlsrc/pbl-met-hierarchy.sml"
neuper@41905
    46
   use    "xmlsrc/thy-hierarchy.sml" 
neuper@41905
    47
   use    "xmlsrc/interface-xml.sml"
neuper@41905
    48
*)        "xmlsrc/xmlsrc"
neuper@41905
    49
neuper@41905
    50
(* use     "Frontend/messages.sml"
neuper@41905
    51
   use     "Frontend/states.sml"
neuper@41905
    52
   use     "Frontend/interface.sml"
neuper@41905
    53
neuper@41905
    54
   use     "print_exn_G.sml"
neuper@41905
    55
*)         "Frontend/Frontend"
bonzai@41918
    56
neuper@42400
    57
(*         "Knowledge/Isac"
neuper@42400
    58
*)
neuper@42400
    59
           "Knowledge/Build_Thydata"
neuper@37906
    60
begin
neuper@41931
    61
neuper@41931
    62
text {*check presence of definitions from directories*}
neuper@41905
    63
ML {* is_reall_dsc; (*from "ProgLang/scrtools.sml" *) *}
neuper@41905
    64
ML {* me; (*from "Interpret/mathengine.sml"*) *}
neuper@41905
    65
ML {* contextthyOK2xml; (*"xmlsrc/interface-xml.sml"*) *}
neuper@41905
    66
ML {* print_exn_unit *}
neuper@41905
    67
ML {* list_rls (*from Atools.thy*) *}
neuper@41905
    68
ML {* eval_occurs_in (*from Atools.thy*) *}
neuper@41905
    69
ML {* @{thm last_thmI} (*from Atools.thy*) *}
neuper@41931
    70
ML {*@{thm Querkraft_Belastung}*}
neuper@41905
    71
neuper@38009
    72
ML {* check_guhs_unique := false; *}
neuper@38015
    73
ML {* tracing "**** isac kernel = math-engine + Knowledge complete ******" *}
neuper@41943
    74
ML {* @{theory "Isac"} *}
neuper@42407
    75
ML {* ! isab_thm_thy *}
neuper@42412
    76
neuper@37906
    77
end