src/ZF/Coind/Map.thy
author paulson
Thu, 31 May 2001 18:28:23 +0200
changeset 11354 9b80fe19407f
parent 11318 6536fb8c9fc6
child 12595 0480d02221b8
permissions -rw-r--r--
examples files start from Main instead of various ZF theories
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     1
(*  Title:      ZF/Coind/Map.thy
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     2
    ID:         $Id$
1478
2b8c2a7547ab expanded tabs
clasohm
parents: 1401
diff changeset
     3
    Author:     Jacob Frost, Cambridge University Computer Laboratory
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     4
    Copyright   1995  University of Cambridge
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     5
*)
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     6
11354
9b80fe19407f examples files start from Main instead of various ZF theories
paulson
parents: 11318
diff changeset
     7
Map = Main +
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
     8
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
     9
constdefs
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 933
diff changeset
    10
  TMap :: [i,i] => i
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    11
   "TMap(A,B) == {m \\<in> Pow(A*Union(B)).\\<forall>a \\<in> A. m``{a} \\<in> B}"
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    12
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 933
diff changeset
    13
  PMap :: [i,i] => i
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    14
   "PMap(A,B) == TMap(A,cons(0,B))"
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    15
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    16
(* Note: 0 \\<in> B ==> TMap(A,B) = PMap(A,B) *)
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    17
  
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 933
diff changeset
    18
  map_emp :: i
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    19
   "map_emp == 0"
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    20
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 933
diff changeset
    21
  map_owr :: [i,i,i]=>i
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    22
   "map_owr(m,a,b) == \\<Sigma>x \\<in> {a} Un domain(m). if x=a then b else m``{x}"
1401
0c439768f45c removed quotes from consts and syntax sections
clasohm
parents: 933
diff changeset
    23
  map_app :: [i,i]=>i
11318
6536fb8c9fc6 X-symbols for ZF
paulson
parents: 6068
diff changeset
    24
   "map_app(m,a) == m``{a}"
915
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    25
  
6dae0daf57b7 New example by Jacob Frost, tidied by lcp
lcp
parents:
diff changeset
    26
end