src/HOL/Library/Library.thy
author obua
Mon, 01 Aug 2005 11:39:33 +0200
changeset 16966 37e34f315057
parent 16908 d374530bfaaa
child 17516 45164074dad4
permissions -rw-r--r--
1. changed configuration variables for linear programming (Cplex_tools): LP_SOLVER is either CPLEX or GLPK CPLEX_PATH is the path to the cplex binary GLPK_PATH is the path to the glpk binary The change makes it possible to switch between glpk and cplex at runtime. 2. moved conflicting list theories out of Library.thy into ROOT.ML

(*<*)
theory Library
imports
  Accessible_Part
  BigO
  Continuity
  EfficientNat
  FuncSet
  Multiset
  NatPair
  Nat_Infinity
  Nested_Environment
  OptionalSugar
  Permutation
  Primes
  Quotient
  While_Combinator
  Word
  Zorn
  Char_ord
begin
end
(*>*)