src/HOL/Library/Library.thy
author avigad
Mon, 25 Jul 2005 18:54:49 +0200
changeset 16908 d374530bfaaa
parent 16109 e8c169d6f191
child 16966 37e34f315057
permissions -rw-r--r--
Added two new theories to HOL/Library: SetsAndFunctions.thy and BigO.thy

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