src/HOL/Library/Library.thy
author berghofe
Wed, 24 Nov 2004 10:28:09 +0100
changeset 15322 c93e6fd5db59
parent 15140 322485b816ac
child 15324 c27165172e30
permissions -rw-r--r--
Added Library/EfficientNat
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
10253
73b46b18c348 "The Supplemental Isabelle/HOL Library";
wenzelm
parents:
diff changeset
     1
(*<*)
15131
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     2
theory Library
15140
322485b816ac import -> imports
nipkow
parents: 15131
diff changeset
     3
imports
15131
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     4
  Accessible_Part
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     5
  Continuity
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     6
  FuncSet
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     7
  List_Prefix
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     8
  Multiset
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     9
  NatPair
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    10
  Nat_Infinity
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    11
  Nested_Environment
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    12
  Permutation
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    13
  Primes
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    14
  Quotient
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    15
  While_Combinator
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    16
  Word
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    17
  Zorn
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    18
begin
10253
73b46b18c348 "The Supplemental Isabelle/HOL Library";
wenzelm
parents:
diff changeset
    19
end
73b46b18c348 "The Supplemental Isabelle/HOL Library";
wenzelm
parents:
diff changeset
    20
(*>*)