allow to load this into "isabelle jedit -l HOL";
authorwenzelm
Tue, 04 Apr 2017 23:21:16 +0200
changeset 65386 e3fb3036a00e
parent 65385 23f36ab9042b
child 65387 5dbe02addca5
child 65391 b5740579cad6
allow to load this into "isabelle jedit -l HOL";
src/ZF/ZF.thy
--- a/src/ZF/ZF.thy	Tue Apr 04 23:12:08 2017 +0200
+++ b/src/ZF/ZF.thy	Tue Apr 04 23:21:16 2017 +0200
@@ -217,7 +217,7 @@
 definition relation :: "i \<Rightarrow> o"  \<comment> \<open>recognizes sets of pairs\<close>
   where "relation(r) == \<forall>z\<in>r. \<exists>x y. z = \<langle>x,y\<rangle>"
 
-definition function :: "i \<Rightarrow> o"  \<comment> \<open>recognizes functions; can have non-pairs\<close>
+definition "function" :: "i \<Rightarrow> o"  \<comment> \<open>recognizes functions; can have non-pairs\<close>
   where "function(r) == \<forall>x y. \<langle>x,y\<rangle> \<in> r \<longrightarrow> (\<forall>y'. \<langle>x,y'\<rangle> \<in> r \<longrightarrow> y = y')"
 
 definition Image :: "[i, i] \<Rightarrow> i"  (infixl "``" 90)  \<comment> \<open>image\<close>