src/HOL/Library/Library.thy
author webertj
Thu, 28 Oct 2004 19:40:22 +0200
changeset 15269 f856f4f3258f
parent 15140 322485b816ac
child 15324 c27165172e30
permissions -rw-r--r--
isatool usedir: ML root file can now be specified (previously hard-coded as ROOT.ML)

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