src/Tools/isac/Knowledge/Atools.thy
branchisac-update-Isa09-2
changeset 37954 4022d670753c
parent 37949 aaf528d3ebd5
child 37959 cc24d0f70544
equal deleted inserted replaced
37953:369b3012f6f6 37954:4022d670753c
     4 
     4 
     5 12345678901234567890123456789012345678901234567890123456789012345678901234567890
     5 12345678901234567890123456789012345678901234567890123456789012345678901234567890
     6         10        20        30        40        50        60        70        80
     6         10        20        30        40        50        60        70        80
     7 *)
     7 *)
     8 
     8 
     9 (*theory Atools imports Descript Typefix begin  ...WOULD BE REQUIRED*)
     9 theory Atools imports Descript Typefix (*...WOULD BE REQUIRED*)
    10 theory Atools imports Complex_Main
    10 (*theory Atools imports Complex_Main*)
    11 (*theory Atools imports "../Knowledge/Descript" "../Knowledge/Typefix" begin*)
    11 (*theory Atools imports "../Knowledge/Descript" "../Knowledge/Typefix" begin*)
    12 uses ("../ProgLang/term.sml")
    12 uses ("../ProgLang/term.sml")
    13 begin
    13 begin
    14 use "../ProgLang/term.sml"
    14 use "../ProgLang/term.sml"
    15 
    15