src/HOL/Library/Library.thy
author wenzelm
Tue, 31 May 2005 11:53:14 +0200
changeset 16123 1381e90c2694
parent 16109 e8c169d6f191
child 16908 d374530bfaaa
permissions -rw-r--r--
Theory.restore_naming;

(*<*)
theory Library
imports
  Accessible_Part
  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
(*>*)