remove intro! attribute from {sinl,sinr}_defined
authorhuffman
Thu, 21 Oct 2010 05:44:38 -0700
changeset 40081 748911a00a51
parent 40080 435f9f5970f8
child 40082 f4be971c5746
remove intro! attribute from {sinl,sinr}_defined
src/HOLCF/Ssum.thy
--- a/src/HOLCF/Ssum.thy	Thu Oct 21 05:35:32 2010 -0700
+++ b/src/HOLCF/Ssum.thy	Thu Oct 21 05:44:38 2010 -0700
@@ -108,10 +108,10 @@
 lemma sinr_defined_iff [simp]: "(sinr\<cdot>x = \<bottom>) = (x = \<bottom>)"
 using sinr_eq [of "x" "\<bottom>"] by simp
 
-lemma sinl_defined [intro!]: "x \<noteq> \<bottom> \<Longrightarrow> sinl\<cdot>x \<noteq> \<bottom>"
+lemma sinl_defined: "x \<noteq> \<bottom> \<Longrightarrow> sinl\<cdot>x \<noteq> \<bottom>"
 by simp
 
-lemma sinr_defined [intro!]: "x \<noteq> \<bottom> \<Longrightarrow> sinr\<cdot>x \<noteq> \<bottom>"
+lemma sinr_defined: "x \<noteq> \<bottom> \<Longrightarrow> sinr\<cdot>x \<noteq> \<bottom>"
 by simp
 
 text {* Compactness *}