src/HOL/Library/Library.thy
author nipkow
Thu, 09 Dec 2004 18:30:59 +0100
changeset 15392 290bc97038c7
parent 15324 c27165172e30
child 15470 7e12ad2f6672
permissions -rw-r--r--
First step in reorganizing Finite_Set

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