src/ZF/Resid/Confluence.thy
changeset 24893 b8ef7afe3a6b
parent 22808 a7daa74e2980
child 35762 af3ff2ba4c54
--- a/src/ZF/Resid/Confluence.thy	Sun Oct 07 15:49:25 2007 +0200
+++ b/src/ZF/Resid/Confluence.thy	Sun Oct 07 21:19:31 2007 +0200
@@ -7,12 +7,13 @@
 
 theory Confluence imports Reduction begin
 
-constdefs
-  confluence    :: "i=>o"
+definition
+  confluence    :: "i=>o"  where
     "confluence(R) ==   
        \<forall>x y. <x,y> \<in> R --> (\<forall>z.<x,z> \<in> R --> (\<exists>u.<y,u> \<in> R & <z,u> \<in> R))"
 
-  strip         :: "o"
+definition
+  strip         :: "o"  where
     "strip == \<forall>x y. (x ===> y) --> 
                     (\<forall>z.(x =1=> z) --> (\<exists>u.(y =1=> u) & (z===>u)))"