src/ZF/Constructible/Relative.thy
changeset 58860 fee7cfa69c50
parent 52458 210bca64b894
child 58871 c399ae4b836f
--- a/src/ZF/Constructible/Relative.thy	Sat Nov 01 11:40:55 2014 +0100
+++ b/src/ZF/Constructible/Relative.thy	Sat Nov 01 14:20:38 2014 +0100
@@ -1336,7 +1336,7 @@
 text{*The assumption @{term "M(A->B)"} is unusual, but essential: in
 all but trivial cases, A->B cannot be expected to belong to @{term M}.*}
 lemma (in M_basic) is_funspace_abs [simp]:
-     "[|M(A); M(B); M(F); M(A->B)|] ==> is_funspace(M,A,B,F) \<longleftrightarrow> F = A->B";
+     "[|M(A); M(B); M(F); M(A->B)|] ==> is_funspace(M,A,B,F) \<longleftrightarrow> F = A->B"
 apply (simp add: is_funspace_def)
 apply (rule iffI)
  prefer 2 apply blast