src/HOL/Library/Library.thy
author kleing
Fri, 24 Jun 2005 03:16:52 +0200
changeset 16558 e97188c6bd71
parent 16109 e8c169d6f191
child 16908 d374530bfaaa
permissions -rw-r--r--
made su[bp]/isu[bp] behave the same as their bsu[bp]..esu[bp] counterparts, properly respect isastylescript now

(*<*)
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
(*>*)