changeset 35416 | d8d7d1b785af |
parent 21324 | a5089fc012b5 |
child 42765 | aec61b60ff7b |
--- a/doc-src/TutorialI/Overview/LNCS/FP1.thy Wed Feb 24 11:55:52 2010 +0100 +++ b/doc-src/TutorialI/Overview/LNCS/FP1.thy Mon Mar 01 13:40:23 2010 +0100 @@ -62,7 +62,7 @@ consts xor :: "bool \<Rightarrow> bool \<Rightarrow> bool" defs xor_def: "xor x y \<equiv> x \<and> \<not>y \<or> \<not>x \<and> y" -constdefs nand :: "bool \<Rightarrow> bool \<Rightarrow> bool" +definition nand :: "bool \<Rightarrow> bool \<Rightarrow> bool" where "nand x y \<equiv> \<not>(x \<and> y)" lemma "\<not> xor x x"