src/ZF/Epsilon.thy
changeset 58860 fee7cfa69c50
parent 46953 2b6e55924af3
child 58871 c399ae4b836f
--- a/src/ZF/Epsilon.thy	Sat Nov 01 11:40:55 2014 +0100
+++ b/src/ZF/Epsilon.thy	Sat Nov 01 14:20:38 2014 +0100
@@ -117,14 +117,14 @@
 done
 
 text{*A transitive set either is empty or contains the empty set.*}
-lemma Transset_0_lemma [rule_format]: "Transset(A) ==> x\<in>A \<longrightarrow> 0\<in>A";
+lemma Transset_0_lemma [rule_format]: "Transset(A) ==> x\<in>A \<longrightarrow> 0\<in>A"
 apply (simp add: Transset_def)
 apply (rule_tac a=x in eps_induct, clarify)
 apply (drule bspec, assumption)
 apply (case_tac "x=0", auto)
 done
 
-lemma Transset_0_disj: "Transset(A) ==> A=0 | 0\<in>A";
+lemma Transset_0_disj: "Transset(A) ==> A=0 | 0\<in>A"
 by (blast dest: Transset_0_lemma)