src/ZF/Finite.thy
author lcp
Fri, 12 Aug 1994 12:51:34 +0200
changeset 516 1957113f0d7d
child 534 cd8bec47e175
permissions -rw-r--r--
installation of new inductive/datatype sections
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
516
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     1
(*  Title: 	ZF/Finite.thy
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     2
    ID:         $Id$
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     3
    Author: 	Lawrence C Paulson, Cambridge University Computer Laboratory
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     4
    Copyright   1994  University of Cambridge
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     5
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     6
Finite powerset operator
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     7
*)
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     8
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
     9
Finite = Arith + 
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    10
consts Fin :: "i=>i"
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    11
inductive
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    12
  domains   "Fin(A)" <= "Pow(A)"
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    13
  intrs
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    14
    emptyI  "0 : Fin(A)"
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    15
    consI   "[| a: A;  b: Fin(A) |] ==> cons(a,b) : Fin(A)"
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    16
  type_intrs "[empty_subsetI, cons_subsetI, PowI]"
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    17
  type_elims "[make_elim PowD]"
1957113f0d7d installation of new inductive/datatype sections
lcp
parents:
diff changeset
    18
end