src/ZF/upair.thy
changeset 76216 9fc34f76b4e8
parent 76215 a642599ffdea
child 79340 3ef7606a0d11
--- a/src/ZF/upair.thy	Tue Sep 27 17:46:52 2022 +0100
+++ b/src/ZF/upair.thy	Tue Sep 27 17:54:20 2022 +0100
@@ -66,7 +66,7 @@
 subsection\<open>Rules for Binary Intersection, Defined via \<^term>\<open>Upair\<close>\<close>
 
 lemma Int_iff [simp]: "c \<in> A \<inter> B \<longleftrightarrow> (c \<in> A \<and> c \<in> B)"
-apply (unfold Int_def)
+  unfolding Int_def
 apply (blast intro: UpairI1 UpairI2 elim: UpairE)
 done
 
@@ -104,7 +104,7 @@
 subsection\<open>Rules for \<^term>\<open>cons\<close>\<close>
 
 lemma cons_iff [simp]: "a \<in> cons(b,A) \<longleftrightarrow> (a=b | a \<in> A)"
-apply (unfold cons_def)
+  unfolding cons_def
 apply (blast intro: UpairI1 UpairI2 elim: UpairE)
 done
 
@@ -152,7 +152,7 @@
 
 lemma the_equality [intro]:
     "\<lbrakk>P(a);  \<And>x. P(x) \<Longrightarrow> x=a\<rbrakk> \<Longrightarrow> (THE x. P(x)) = a"
-apply (unfold the_def)
+  unfolding the_def
 apply (fast dest: subst)
 done
 
@@ -171,7 +171,7 @@
 
 (*If it's "undefined", it's zero!*)
 lemma the_0: "\<not> (\<exists>!x. P(x)) \<Longrightarrow> (THE x. P(x))=0"
-apply (unfold the_def)
+  unfolding the_def
 apply (blast elim!: ReplaceE)
 done