src/HOL/GroupTheory/PiSets.thy
author paulson
Tue, 13 Aug 2002 17:42:34 +0200
changeset 13496 6f0c57def6d5
parent 12459 6978ab7cac64
permissions -rw-r--r--
In ZF/Constructible, moved many results from Satisfies_absolute, etc., to the new theory Internalize.thy

(*  Title:      HOL/ex/PiSets.thy
    ID:         $Id$
    Author:     Florian Kammueller, University of Cambridge

The bijection between elements of the Pi set and functional graphs
*)

PiSets = Group +

constdefs
(* bijection between Pi_sig and Pi_=> *)
  PiBij :: "['a set, 'a => 'b set, 'a => 'b] => ('a * 'b) set"
    "PiBij A B == %f: Pi A B. {(x, y). x: A & y = f x}"

  Graph ::  "['a set, 'a => 'b set] => ('a * 'b) set set"
   "Graph A B == {f. f \\<in> Pow(Sigma A B) & (\\<forall>x\\<in>A. \\<exists>!y. (x, y) \\<in> f)}"

end