src/ZF/ZF.thy
changeset 46972 ef6fc1a0884d
parent 46907 eea3eb057fea
child 48462 424fd5364f15
--- a/src/ZF/ZF.thy	Fri Mar 16 21:59:19 2012 +0100
+++ b/src/ZF/ZF.thy	Fri Mar 16 22:22:05 2012 +0100
@@ -14,11 +14,10 @@
 typedecl i
 arities  i :: "term"
 
-consts
-
-  zero        :: "i"                  ("0")   --{*the empty set*}
-  Pow         :: "i => i"                     --{*power sets*}
-  Inf         :: "i"                          --{*infinite set*}
+axiomatization
+  zero :: "i"  ("0")   --{*the empty set*}  and
+  Pow :: "i => i"  --{*power sets*}  and
+  Inf :: "i"  --{*infinite set*}
 
 text {*Bounded Quantifiers *}
 consts
@@ -26,13 +25,12 @@
   Bex   :: "[i, i => o] => o"
 
 text {*General Union and Intersection *}
-consts
-  Union :: "i => i"
-  Inter :: "i => i"
+axiomatization Union :: "i => i"
+consts Inter :: "i => i"
 
 text {*Variations on Replacement *}
+axiomatization PrimReplace :: "[i, [i, i] => o] => i"
 consts
-  PrimReplace :: "[i, [i, i] => o] => i"
   Replace     :: "[i, [i, i] => o] => i"
   RepFun      :: "[i, i => i] => i"
   Collect     :: "[i, i => o] => i"
@@ -196,9 +194,6 @@
   "_pattern"  :: "patterns => pttrn"         ("\<langle>_\<rangle>")
 
 
-finalconsts
-  0 Pow Inf Union PrimReplace mem
-
 defs  (* Bounded Quantifiers *)
   Ball_def:      "Ball(A, P) == \<forall>x. x\<in>A \<longrightarrow> P(x)"
   Bex_def:       "Bex(A, P) == \<exists>x. x\<in>A & P(x)"