src/HOL/Set.thy
author paulson
Fri, 30 Oct 1998 10:45:08 +0100
changeset 5780 0187f936685a
parent 5492 d9fc3457554e
child 5931 325300576da7
permissions -rw-r--r--
Moved "instance set:...{power} from Set.thy to RelPow.thy, where is is needed
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     1
(*  Title:      HOL/Set.thy
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     2
    ID:         $Id$
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     3
    Author:     Tobias Nipkow
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     4
    Copyright   1993  University of Cambridge
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     5
*)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     6
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     7
Set = Ord +
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
     8
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
     9
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    10
(** Core syntax **)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    11
3947
eb707467f8c5 adapted to qualified names;
wenzelm
parents: 3842
diff changeset
    12
global
eb707467f8c5 adapted to qualified names;
wenzelm
parents: 3842
diff changeset
    13
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    14
types
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    15
  'a set
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    16
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    17
arities
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    18
  set :: (term) term
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    19
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    20
instance
5780
0187f936685a Moved "instance set:...{power} from Set.thy to RelPow.thy, where is is needed
paulson
parents: 5492
diff changeset
    21
  set :: (term) {ord, minus}
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    22
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
    23
syntax
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
    24
  "op :"        :: ['a, 'a set] => bool             ("op :")
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
    25
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    26
consts
1370
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    27
  "{}"          :: 'a set                           ("{}")
4159
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    28
  UNIV          :: 'a set
1370
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    29
  insert        :: ['a, 'a set] => 'a set
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    30
  Collect       :: ('a => bool) => 'a set               (*comprehension*)
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    31
  Int           :: ['a set, 'a set] => 'a set       (infixl 70)
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    32
  Un            :: ['a set, 'a set] => 'a set       (infixl 65)
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    33
  UNION, INTER  :: ['a set, 'a => 'b set] => 'b set     (*general*)
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    34
  Union, Inter  :: (('a set) set) => 'a set             (*of a set*)
1370
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    35
  Pow           :: 'a set => 'a set set                 (*powerset*)
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    36
  range         :: ('a => 'b) => 'b set                 (*of function*)
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    37
  Ball, Bex     :: ['a set, 'a => bool] => bool         (*bounded quantifiers*)
1962
e60a230da179 Corrected associativity: must be to right, as the type dictatess
paulson
parents: 1883
diff changeset
    38
  "``"          :: ['a => 'b, 'a set] => ('b set)   (infixr 90)
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    39
  (*membership*)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    40
  "op :"        :: ['a, 'a set] => bool             ("(_/ : _)" [50, 51] 50)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    41
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    42
5492
d9fc3457554e From Compl(A) to -A
paulson
parents: 5254
diff changeset
    43
(*For compatibility: DELETE after one release*)
d9fc3457554e From Compl(A) to -A
paulson
parents: 5254
diff changeset
    44
syntax Compl :: ('a set) => 'a set   (*complement*)
d9fc3457554e From Compl(A) to -A
paulson
parents: 5254
diff changeset
    45
translations "Compl A"  => "- A"
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    46
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    47
(** Additional concrete syntax **)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    48
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    49
syntax
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    50
5492
d9fc3457554e From Compl(A) to -A
paulson
parents: 5254
diff changeset
    51
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    52
  (* Infix syntax for non-membership *)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    53
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
    54
  "op ~:"       :: ['a, 'a set] => bool               ("op ~:")
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    55
  "op ~:"       :: ['a, 'a set] => bool               ("(_/ ~: _)" [50, 51] 50)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    56
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    57
  "@Finset"     :: args => 'a set                     ("{(_)}")
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    58
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    59
  "@Coll"       :: [pttrn, bool] => 'a set            ("(1{_./ _})")
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    60
  "@SetCompr"   :: ['a, idts, bool] => 'a set         ("(1{_ |/_./ _})")
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    61
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    62
  (* Big Intersection / Union *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    63
4159
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    64
  INTER1        :: [pttrns, 'a => 'b set] => 'b set   ("(3INT _./ _)" 10)
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    65
  UNION1        :: [pttrns, 'a => 'b set] => 'b set   ("(3UN _./ _)" 10)
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    66
1370
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    67
  "@INTER"      :: [pttrn, 'a set, 'b set] => 'b set  ("(3INT _:_./ _)" 10)
7361ac9b024d removed quotes from types in consts and syntax sections
clasohm
parents: 1273
diff changeset
    68
  "@UNION"      :: [pttrn, 'a set, 'b set] => 'b set  ("(3UN _:_./ _)" 10)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    69
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    70
  (* Bounded Quantifiers *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    71
2368
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
    72
  "@Ball"       :: [pttrn, 'a set, bool] => bool      ("(3! _:_./ _)" [0, 0, 10] 10)
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
    73
  "@Bex"        :: [pttrn, 'a set, bool] => bool      ("(3? _:_./ _)" [0, 0, 10] 10)
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
    74
  "*Ball"       :: [pttrn, 'a set, bool] => bool      ("(3ALL _:_./ _)" [0, 0, 10] 10)
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
    75
  "*Bex"        :: [pttrn, 'a set, bool] => bool      ("(3EX _:_./ _)" [0, 0, 10] 10)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    76
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    77
translations
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
    78
  "range f"     == "f``UNIV"
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    79
  "x ~: y"      == "~ (x : y)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    80
  "{x, xs}"     == "insert x {xs}"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    81
  "{x}"         == "insert x {}"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    82
  "{x. P}"      == "Collect (%x. P)"
4159
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    83
  "UN x y. B"   == "UN x. UN y. B"
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    84
  "UN x. B"     == "UNION UNIV (%x. B)"
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    85
  "INT x y. B"   == "INT x. INT y. B"
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    86
  "INT x. B"    == "INTER UNIV (%x. B)"
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
    87
  "UN x:A. B"   == "UNION A (%x. B)"
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    88
  "INT x:A. B"  == "INTER A (%x. B)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    89
  "! x:A. P"    == "Ball A (%x. P)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    90
  "? x:A. P"    == "Bex A (%x. P)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    91
  "ALL x:A. P"  => "Ball A (%x. P)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    92
  "EX x:A. P"   => "Bex A (%x. P)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    93
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
    94
syntax ("" output)
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
    95
  "_setle"      :: ['a set, 'a set] => bool           ("op <=")
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
    96
  "_setle"      :: ['a set, 'a set] => bool           ("(_/ <= _)" [50, 51] 50)
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
    97
  "_setless"    :: ['a set, 'a set] => bool           ("op <")
2684
9781d63ef063 added proper subset symbols syntax;
wenzelm
parents: 2412
diff changeset
    98
  "_setless"    :: ['a set, 'a set] => bool           ("(_/ < _)" [50, 51] 50)
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
    99
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   100
syntax (symbols)
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
   101
  "_setle"      :: ['a set, 'a set] => bool           ("op \\<subseteq>")
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
   102
  "_setle"      :: ['a set, 'a set] => bool           ("(_/ \\<subseteq> _)" [50, 51] 50)
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
   103
  "_setless"    :: ['a set, 'a set] => bool           ("op \\<subset>")
2684
9781d63ef063 added proper subset symbols syntax;
wenzelm
parents: 2412
diff changeset
   104
  "_setless"    :: ['a set, 'a set] => bool           ("(_/ \\<subset> _)" [50, 51] 50)
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   105
  "op Int"      :: ['a set, 'a set] => 'a set         (infixl "\\<inter>" 70)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   106
  "op Un"       :: ['a set, 'a set] => 'a set         (infixl "\\<union>" 65)
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
   107
  "op :"        :: ['a, 'a set] => bool               ("op \\<in>")
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   108
  "op :"        :: ['a, 'a set] => bool               ("(_/ \\<in> _)" [50, 51] 50)
3820
46b255e140dc fixed infix syntax;
wenzelm
parents: 3370
diff changeset
   109
  "op ~:"       :: ['a, 'a set] => bool               ("op \\<notin>")
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   110
  "op ~:"       :: ['a, 'a set] => bool               ("(_/ \\<notin> _)" [50, 51] 50)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   111
  "UN "         :: [idts, bool] => bool               ("(3\\<Union> _./ _)" 10)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   112
  "INT "        :: [idts, bool] => bool               ("(3\\<Inter> _./ _)" 10)
4159
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
   113
  "UNION1"      :: [pttrn, 'b set] => 'b set          ("(3\\<Union> _./ _)" 10)
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
   114
  "INTER1"      :: [pttrn, 'b set] => 'b set          ("(3\\<Inter> _./ _)" 10)
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   115
  "@UNION"      :: [pttrn, 'a set, 'b set] => 'b set  ("(3\\<Union> _\\<in>_./ _)" 10)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   116
  "@INTER"      :: [pttrn, 'a set, 'b set] => 'b set  ("(3\\<Inter> _\\<in>_./ _)" 10)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   117
  Union         :: (('a set) set) => 'a set           ("\\<Union> _" [90] 90)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   118
  Inter         :: (('a set) set) => 'a set           ("\\<Inter> _" [90] 90)
2368
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
   119
  "@Ball"       :: [pttrn, 'a set, bool] => bool      ("(3\\<forall> _\\<in>_./ _)" [0, 0, 10] 10)
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
   120
  "@Bex"        :: [pttrn, 'a set, bool] => bool      ("(3\\<exists> _\\<in>_./ _)" [0, 0, 10] 10)
2372
a2999e19703b fixed alternative quantifier symbol syntax;
wenzelm
parents: 2368
diff changeset
   121
a2999e19703b fixed alternative quantifier symbol syntax;
wenzelm
parents: 2368
diff changeset
   122
syntax (symbols output)
2368
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
   123
  "*Ball"       :: [pttrn, 'a set, bool] => bool      ("(3\\<forall> _\\<in>_./ _)" [0, 0, 10] 10)
d394336997cf fixed pris of binder syntax;
wenzelm
parents: 2261
diff changeset
   124
  "*Bex"        :: [pttrn, 'a set, bool] => bool      ("(3\\<exists> _\\<in>_./ _)" [0, 0, 10] 10)
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   125
2412
025e80ed698d fixed \<subseteq> input;
wenzelm
parents: 2393
diff changeset
   126
translations
2965
afbda7e26f15 improved translations for subset symbols syntax: constraints;
wenzelm
parents: 2912
diff changeset
   127
  "op \\<subseteq>" => "op <= :: [_ set, _ set] => bool"
afbda7e26f15 improved translations for subset symbols syntax: constraints;
wenzelm
parents: 2912
diff changeset
   128
  "op \\<subset>" => "op <  :: [_ set, _ set] => bool"
2412
025e80ed698d fixed \<subseteq> input;
wenzelm
parents: 2393
diff changeset
   129
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   130
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   131
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   132
(** Rules and definitions **)
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   133
3947
eb707467f8c5 adapted to qualified names;
wenzelm
parents: 3842
diff changeset
   134
local
eb707467f8c5 adapted to qualified names;
wenzelm
parents: 3842
diff changeset
   135
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   136
rules
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   137
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   138
  (* Isomorphisms between Predicates and Sets *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   139
3842
b55686a7b22c fixed dots;
wenzelm
parents: 3820
diff changeset
   140
  mem_Collect_eq    "(a : {x. P(x)}) = P(a)"
b55686a7b22c fixed dots;
wenzelm
parents: 3820
diff changeset
   141
  Collect_mem_eq    "{x. x:A} = A"
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   142
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   143
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   144
defs
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   145
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   146
  Ball_def      "Ball A P       == ! x. x:A --> P(x)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   147
  Bex_def       "Bex A P        == ? x. x:A & P(x)"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   148
  subset_def    "A <= B         == ! x:A. x:B"
3222
726a9b069947 Distributed Psubset stuff to basic set theory files, incl Finite.
nipkow
parents: 2965
diff changeset
   149
  psubset_def   "A < B          == (A::'a set) <= B & ~ A=B"
5492
d9fc3457554e From Compl(A) to -A
paulson
parents: 5254
diff changeset
   150
  Compl_def     "- A            == {x. ~x:A}"
3842
b55686a7b22c fixed dots;
wenzelm
parents: 3820
diff changeset
   151
  Un_def        "A Un B         == {x. x:A | x:B}"
b55686a7b22c fixed dots;
wenzelm
parents: 3820
diff changeset
   152
  Int_def       "A Int B        == {x. x:A & x:B}"
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   153
  set_diff_def  "A - B          == {x. x:A & ~x:B}"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   154
  INTER_def     "INTER A B      == {y. ! x:A. y: B(x)}"
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   155
  UNION_def     "UNION A B      == {y. ? x:A. y: B(x)}"
2393
651fce76c86c adaptions for symbol font
oheimb
parents: 2388
diff changeset
   156
  Inter_def     "Inter S        == (INT x:S. x)"
651fce76c86c adaptions for symbol font
oheimb
parents: 2388
diff changeset
   157
  Union_def     "Union S        == (UN x:S. x)"
651fce76c86c adaptions for symbol font
oheimb
parents: 2388
diff changeset
   158
  Pow_def       "Pow A          == {B. B <= A}"
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   159
  empty_def     "{}             == {x. False}"
4159
4aff9b7e5597 UNIV now a constant; UNION1, INTER1 now translations and no longer have
paulson
parents: 4151
diff changeset
   160
  UNIV_def      "UNIV           == {x. True}"
3842
b55686a7b22c fixed dots;
wenzelm
parents: 3820
diff changeset
   161
  insert_def    "insert a B     == {x. x=a} Un B"
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   162
  image_def     "f``A           == {y. ? x:A. y=f(x)}"
1273
6960ec882bca added 8bit pragmas
regensbu
parents: 1068
diff changeset
   163
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   164
end
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   165
2261
d926157c0a6a added "op :", "op ~:" syntax;
wenzelm
parents: 2006
diff changeset
   166
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   167
ML
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   168
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   169
local
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   170
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
   171
(* Set inclusion *)
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
   172
4151
5c19cd418c33 adapted typed_print_translation;
wenzelm
parents: 3947
diff changeset
   173
fun le_tr' _ (*op <=*) (Type ("fun", (Type ("set", _) :: _))) ts =
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
   174
      list_comb (Syntax.const "_setle", ts)
4151
5c19cd418c33 adapted typed_print_translation;
wenzelm
parents: 3947
diff changeset
   175
  | le_tr' _ (*op <=*) _ _ = raise Match;
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
   176
4151
5c19cd418c33 adapted typed_print_translation;
wenzelm
parents: 3947
diff changeset
   177
fun less_tr' _ (*op <*) (Type ("fun", (Type ("set", _) :: _))) ts =
2684
9781d63ef063 added proper subset symbols syntax;
wenzelm
parents: 2412
diff changeset
   178
      list_comb (Syntax.const "_setless", ts)
4151
5c19cd418c33 adapted typed_print_translation;
wenzelm
parents: 3947
diff changeset
   179
  | less_tr' _ (*op <*) _ _ = raise Match;
2684
9781d63ef063 added proper subset symbols syntax;
wenzelm
parents: 2412
diff changeset
   180
2388
d1f0505fc602 added set inclusion symbol syntax;
wenzelm
parents: 2372
diff changeset
   181
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   182
(* Translates between { e | x1..xn. P} and {u. ? x1..xn. u=e & P}      *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   183
(* {y. ? x1..xn. y = e & P} is only translated if [0..n] subset bvs(e) *)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   184
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   185
val ex_tr = snd(mk_binder_tr("? ","Ex"));
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   186
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   187
fun nvars(Const("_idts",_) $ _ $ idts) = nvars(idts)+1
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   188
  | nvars(_) = 1;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   189
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   190
fun setcompr_tr[e,idts,b] =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   191
  let val eq = Syntax.const("op =") $ Bound(nvars(idts)) $ e
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   192
      val P = Syntax.const("op &") $ eq $ b
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   193
      val exP = ex_tr [idts,P]
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   194
  in Syntax.const("Collect") $ Abs("",dummyT,exP) end;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   195
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   196
val ex_tr' = snd(mk_binder_tr' ("Ex","DUMMY"));
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   197
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   198
fun setcompr_tr'[Abs(_,_,P)] =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   199
  let fun ok(Const("Ex",_)$Abs(_,_,P),n) = ok(P,n+1)
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   200
        | ok(Const("op &",_) $ (Const("op =",_) $ Bound(m) $ e) $ _, n) =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   201
            if n>0 andalso m=n andalso
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   202
              ((0 upto (n-1)) subset add_loose_bnos(e,0,[]))
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   203
            then () else raise Match
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   204
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   205
      fun tr'(_ $ abs) =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   206
        let val _ $ idts $ (_ $ (_ $ _ $ e) $ Q) = ex_tr'[abs]
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   207
        in Syntax.const("@SetCompr") $ e $ idts $ Q end
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   208
  in ok(P,0); tr'(P) end;
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   209
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   210
in
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   211
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   212
val parse_translation = [("@SetCompr", setcompr_tr)];
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   213
val print_translation = [("Collect", setcompr_tr')];
2684
9781d63ef063 added proper subset symbols syntax;
wenzelm
parents: 2412
diff changeset
   214
val typed_print_translation = [("op <=", le_tr'), ("op <", less_tr')];
923
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   215
val print_ast_translation =
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   216
  map HOL.alt_ast_tr' [("@Ball", "*Ball"), ("@Bex", "*Bex")];
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   217
ff1574a81019 new version of HOL with curried function application
clasohm
parents:
diff changeset
   218
end;