changeset 17555 | 23c4a349feff |
parent 16417 | 9bc16273c2d4 |
child 27015 | f8537d69f514 |
--- a/doc-src/TutorialI/Ifexpr/Ifexpr.thy Wed Sep 21 13:28:44 2005 +0200 +++ b/doc-src/TutorialI/Ifexpr/Ifexpr.thy Wed Sep 21 14:00:28 2005 +0200 @@ -36,7 +36,7 @@ values: *} -consts value :: "boolex \<Rightarrow> (nat \<Rightarrow> bool) \<Rightarrow> bool"; +consts "value" :: "boolex \<Rightarrow> (nat \<Rightarrow> bool) \<Rightarrow> bool"; primrec "value (Const b) env = b" "value (Var x) env = env x"