src/Tools/isac/BaseDefinitions/BaseDefinitions.thy
author Walther Neuper <walther.neuper@jku.at>
Tue, 28 Apr 2020 15:31:49 +0200
changeset 59914 ab5bd5c37e13
parent 59911 ff30cec13f4f
child 59918 58d9fcc5a712
permissions -rw-r--r--
assign code from Rtools to appropriate struct.s
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@59889
     9
  ML_file calcelems.sml
walther@59659
    10
  ML_file termC.sml
walther@59911
    11
  ML_file substitution.sml
walther@59659
    12
  ML_file contextC.sml
walther@59659
    13
  ML_file environment.sml
walther@59630
    14
wneuper@59586
    15
ML \<open>
wneuper@59586
    16
\<close> ML \<open>
walther@59914
    17
Library.distinct: ('a * 'a -> bool) -> 'a list -> 'a list
wneuper@59586
    18
\<close> ML \<open>
wneuper@59586
    19
\<close>
wneuper@59586
    20
end