src/HOL/GroupTheory/PiSets.thy
changeset 13583 5fcc8bf538ee
parent 13582 a246a0a52dfb
child 13584 3736cf381e15
--- a/src/HOL/GroupTheory/PiSets.thy	Wed Sep 25 11:23:26 2002 +0200
+++ /dev/null	Thu Jan 01 00:00:00 1970 +0000
@@ -1,18 +0,0 @@
-(*  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