src/HOL/Library/FuncSet.thy
changeset 73348 65c45cba3f54
parent 73346 00e0f7724c06
child 73932 fd21b4a93043
--- a/src/HOL/Library/FuncSet.thy	Mon Mar 01 14:47:08 2021 +0000
+++ b/src/HOL/Library/FuncSet.thy	Mon Mar 01 17:59:17 2021 +0000
@@ -73,7 +73,7 @@
 
 lemma Pi_eq_empty[simp]: "(\<Pi> x \<in> A. B x) = {} \<longleftrightarrow> (\<exists>x\<in>A. B x = {})"
 proof -
-  have "\<exists>x\<in>A. B x = {}" if "\<And>f. \<exists>y. y \<in> A \<and> f y \<notin> B y" 
+  have "\<exists>x\<in>A. B x = {}" if "\<And>f. \<exists>y. y \<in> A \<and> f y \<notin> B y"
     using that [of "\<lambda>u. SOME y. y \<in> B u"] some_in_eq by blast
   then show ?thesis
     by force
@@ -432,7 +432,7 @@
 lemma PiE_iff: "f \<in> Pi\<^sub>E I X \<longleftrightarrow> (\<forall>i\<in>I. f i \<in> X i) \<and> f \<in> extensional I"
   by (simp add: PiE_def Pi_iff)
 
-lemma restrict_PiE_iff [simp]: "restrict f I \<in> Pi\<^sub>E I X \<longleftrightarrow> (\<forall>i \<in> I. f i \<in> X i)"
+lemma restrict_PiE_iff: "restrict f I \<in> Pi\<^sub>E I X \<longleftrightarrow> (\<forall>i \<in> I. f i \<in> X i)"
   by (simp add: PiE_iff)
 
 lemma ext_funcset_to_sing_iff [simp]: "A \<rightarrow>\<^sub>E {a} = {\<lambda>x\<in>A. a}"
@@ -537,7 +537,7 @@
     by auto
 qed
 
-lemma PiE_singleton: 
+lemma PiE_singleton:
   assumes "f \<in> extensional A"
   shows   "PiE A (\<lambda>x. {f x}) = {f}"
 proof -