Got rid of the [iff], which was effectively inserting converseD
authorpaulson
Wed, 23 Apr 2003 13:06:36 +0200
changeset 13919 17d0e17c8efe
parent 13918 2134ed516b1b
child 13920 9d542c96e855
Got rid of the [iff], which was effectively inserting converseD
src/ZF/equalities.thy
--- a/src/ZF/equalities.thy	Wed Apr 23 00:14:55 2003 +0200
+++ b/src/ZF/equalities.thy	Wed Apr 23 13:06:36 2003 +0200
@@ -70,10 +70,10 @@
 
 subsection{*Converse of a Relation*}
 
-lemma converse_iff [iff]: "<a,b>: converse(r) <-> <b,a>:r"
+lemma converse_iff [simp]: "<a,b>: converse(r) <-> <b,a>:r"
 by (unfold converse_def, blast)
 
-lemma converseI: "<a,b>:r ==> <b,a>:converse(r)"
+lemma converseI [intro!]: "<a,b>:r ==> <b,a>:converse(r)"
 by (unfold converse_def, blast)
 
 lemma converseD: "<a,b> : converse(r) ==> <b,a> : r"