src/HOL/ZF/HOLZF.thy
changeset 67443 3abf6a722518
parent 63901 4ce989e962e0
child 67613 ce654b0e6d69
equal deleted inserted replaced
67442:f075640b8868 67443:3abf6a722518
   186   by (auto simp add: union_def Sum Upair)
   186   by (auto simp add: union_def Sum Upair)
   187 
   187 
   188 definition Field :: "ZF \<Rightarrow> ZF" where
   188 definition Field :: "ZF \<Rightarrow> ZF" where
   189   "Field A == union (Domain A) (Range A)"
   189   "Field A == union (Domain A) (Range A)"
   190 
   190 
   191 definition app :: "ZF \<Rightarrow> ZF => ZF" (infixl "\<acute>" 90) \<comment>\<open>function application\<close> where
   191 definition app :: "ZF \<Rightarrow> ZF => ZF" (infixl "\<acute>" 90) \<comment> \<open>function application\<close> where
   192   "f \<acute> x == (THE y. Elem (Opair x y) f)"
   192   "f \<acute> x == (THE y. Elem (Opair x y) f)"
   193 
   193 
   194 definition isFun :: "ZF \<Rightarrow> bool" where
   194 definition isFun :: "ZF \<Rightarrow> bool" where
   195   "isFun f == (! x y1 y2. Elem (Opair x y1) f & Elem (Opair x y2) f \<longrightarrow> y1 = y2)"
   195   "isFun f == (! x y1 y2. Elem (Opair x y1) f & Elem (Opair x y2) f \<longrightarrow> y1 = y2)"
   196 
   196