src/HOL/Library/Library.thy
author paulson
Mon, 24 Nov 2003 15:33:07 +0100
changeset 14266 08b34c902618
parent 14127 40a4768c8e0b
child 14365 3d4df8c166ae
permissions -rw-r--r--
conversion of integers to use Ring_and_Field;
new lemmas for Ring_and_Field
wenzelm@10253
     1
(*<*)
wenzelm@10253
     2
theory Library =
wenzelm@10332
     3
  Quotient +
oheimb@11349
     4
  Nat_Infinity +
wenzelm@10619
     5
  Rational_Numbers +
wenzelm@10616
     6
  List_Prefix +
wenzelm@10943
     7
  Nested_Environment +
wenzelm@10253
     8
  Accessible_Part +
oheimb@11349
     9
  Continuity +
wenzelm@10253
    10
  Multiset +
wenzelm@11055
    11
  Permutation +
paulson@14127
    12
  NatPair +
wenzelm@11368
    13
  Primes +
nipkow@10984
    14
  While_Combinator:
wenzelm@10253
    15
end
wenzelm@10253
    16
(*>*)