src/Tools/isac/Knowledge/Vect.thy
author Walther Neuper <wneuper@ist.tugraz.at>
Wed, 13 Jan 2016 14:37:27 +0100
changeset 59206 ebf4a8a63371
parent 37992 351a9e94c38d
child 59427 d7a39d815afa
permissions -rw-r--r--
cleanup theory imports, part 1

# Cleanup is triggered by failing session Protocol2015, which gives:
No such file: "/usr/local/isabisac/src/Tools/isac/Complex_Main.thy"
The error(s) above occurred for theory "Complex_Main"
(required by "Protocol" via "Build_Thydata" via "Isac" via "Frontend" via "xmlsrc" via "Interpret" via "ProgLang" via "Script" via "Tools" via "ListC" via "KEStore") (line 6 of "/usr/local/isabisac/src/Tools/isac/KEStore.thy")
No such file: "/usr/local/isabisac/src/Tools/isac/Knowledge/Real.thy"
:
:
# The newly introduced imports "~~/..." avoid the above kind of errors.
# However, these errors still remain:
Build started for Isabelle/Protocol2015 ...
Building Protocol2015 ...
Protocol2015: theory Classy
Protocol2015: theory Code_Generator
:
Protocol2015: theory Taylor
Protocol2015: theory Complex_Main
Protocol2015: theory KEStore
Protocol2015: theory ListC
Protocol2015 FAILED
*** Failed to load theory "RootRatEq" (unresolved "LinEq", "RatEq", "RootEq", "RootRat")
*** Failed to load theory "Partial_Fractions" (unresolved "RootRatEq")
:
:
wneuper@59206
     1
theory Vect imports "~~/src/HOL/Real" begin
neuper@37906
     2
neuper@37906
     3
end