src/HOL/Library/Library.thy
author nipkow
Wed, 26 Jan 2005 16:39:44 +0100
changeset 15470 7e12ad2f6672
parent 15324 c27165172e30
child 15731 29ae73d8a84e
permissions -rw-r--r--
added OptionalSugar
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
15324
c27165172e30 Added EfficientNat
berghofe
parents: 15140
diff changeset
     6
  EfficientNat
15131
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     7
  FuncSet
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     8
  List_Prefix
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
     9
  Multiset
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    10
  NatPair
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    11
  Nat_Infinity
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    12
  Nested_Environment
15470
7e12ad2f6672 added OptionalSugar
nipkow
parents: 15324
diff changeset
    13
  OptionalSugar
15131
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    14
  Permutation
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    15
  Primes
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    16
  Quotient
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    17
  While_Combinator
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    18
  Word
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    19
  Zorn
c69542757a4d New theory header syntax.
nipkow
parents: 14706
diff changeset
    20
begin
10253
73b46b18c348 "The Supplemental Isabelle/HOL Library";
wenzelm
parents:
diff changeset
    21
end
73b46b18c348 "The Supplemental Isabelle/HOL Library";
wenzelm
parents:
diff changeset
    22
(*>*)