src/HOL/Library/Library.thy
author obua
Sun, 29 May 2005 12:41:40 +0200
changeset 16109 e8c169d6f191
parent 15731 29ae73d8a84e
child 16908 d374530bfaaa
permissions -rw-r--r--
Removes an inconsistent definition from Library.thy , so that the lexical order is the standard order for lists. The prefix order is not built any more.

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