doc-src/TutorialI/Sets/Relations.thy
changeset 26806 40b411ec05aa
parent 16417 9bc16273c2d4
child 36745 403585a89772
--- a/doc-src/TutorialI/Sets/Relations.thy	Wed May 07 10:56:58 2008 +0200
+++ b/doc-src/TutorialI/Sets/Relations.thy	Wed May 07 10:57:19 2008 +0200
@@ -151,7 +151,7 @@
 text{*Pow, Inter too little used*}
 
 lemma "(A \<subset> B) = (A \<subseteq> B \<and> A \<noteq> B)"
-apply (simp add: psubset_def)
+apply (simp add: psubset_eq)
 done
 
 end