doc-src/TutorialI/Sets/Functions.thy
changeset 39795 9e59b4c11039
parent 36745 403585a89772
child 42637 381fdcab0f36
--- a/doc-src/TutorialI/Sets/Functions.thy	Thu Sep 30 08:50:45 2010 +0200
+++ b/doc-src/TutorialI/Sets/Functions.thy	Thu Sep 30 09:31:07 2010 +0200
@@ -66,20 +66,18 @@
 \rulename{o_inv_distrib}
 *}
 
-
-
 text{*
 small sample proof
 
 @{thm[display] ext[no_vars]}
 \rulename{ext}
 
-@{thm[display] expand_fun_eq[no_vars]}
-\rulename{expand_fun_eq}
+@{thm[display] fun_eq_iff[no_vars]}
+\rulename{fun_eq_iff}
 *}
 
 lemma "inj f \<Longrightarrow> (f o g = f o h) = (g = h)";
-  apply (simp add: expand_fun_eq inj_on_def)
+  apply (simp add: fun_eq_iff inj_on_def)
   apply (auto)
   done