src/Tools/isac/BaseDefinitions/BaseDefinitions.thy
author wneuper <walther.neuper@jku.at>
Tue, 10 Aug 2021 11:01:18 +0200
changeset 60360 49680d595342
parent 60333 7c76b8278a9f
child 60405 d4ebe139100d
permissions -rw-r--r--
eliminate ThyC.to_ctxt, use Proof_Context.init_global inline
walther@59866
     1
(* Title:  "BaseDefinitions/BaseDefinitions.thy"
wneuper@59586
     2
   Author: Walther Neuper 190823
wneuper@59586
     3
   (c) due to copyright terms
walther@59866
     4
walther@59887
     5
Know_Store holds Theory_Data (problems, methods, etc) and requires respective definitions.
wneuper@59586
     6
*)
walther@59887
     7
theory BaseDefinitions imports Know_Store
wneuper@59586
     8
begin
walther@59659
     9
  ML_file termC.sml
walther@59911
    10
  ML_file substitution.sml
walther@59659
    11
  ML_file contextC.sml
walther@59659
    12
  ML_file environment.sml
walther@59630
    13
wneuper@59586
    14
ML \<open>
wneuper@59586
    15
\<close> ML \<open>
walther@60317
    16
\<close> ML \<open>
wneuper@59586
    17
\<close>
wneuper@59586
    18
end