doc-src/TutorialI/Misc/simp.thy
changeset 27027 63f0b638355c
parent 20212 f4a8b4e2fb29
child 35992 78674c6018ca
--- a/doc-src/TutorialI/Misc/simp.thy	Fri May 30 17:03:37 2008 +0200
+++ b/doc-src/TutorialI/Misc/simp.thy	Fri May 30 17:52:10 2008 +0200
@@ -161,8 +161,8 @@
 
 For example, given *}
 
-constdefs xor :: "bool \<Rightarrow> bool \<Rightarrow> bool"
-         "xor A B \<equiv> (A \<and> \<not>B) \<or> (\<not>A \<and> B)"
+definition xor :: "bool \<Rightarrow> bool \<Rightarrow> bool" where
+"xor A B \<equiv> (A \<and> \<not>B) \<or> (\<not>A \<and> B)"
 
 text{*\noindent
 we may want to prove