src/HOL/Library/Library.thy
author wenzelm
Fri, 03 Nov 2000 21:35:36 +0100
changeset 10389 c7d8901ab269
parent 10332 b4f7f8693f8e
child 10481 9efb2fd5399e
permissions -rw-r--r--
proper setup of "parallel"; removed unused rules;

(*<*)
theory Library =
  List_Prefix +
  Quotient +
  Accessible_Part +
  Multiset +
  While_Combinator + While_Combinator_Example:
end
(*>*)