doc-src/TutorialI/Inductive/Advanced.thy
changeset 39795 9e59b4c11039
parent 32891 d403b99287ff
child 43564 9864182c6bad
--- a/doc-src/TutorialI/Inductive/Advanced.thy	Thu Sep 30 08:50:45 2010 +0200
+++ b/doc-src/TutorialI/Inductive/Advanced.thy	Thu Sep 30 09:31:07 2010 +0200
@@ -1,4 +1,3 @@
-(* ID:         $Id$ *)
 (*<*)theory Advanced imports Even uses "../../antiquote_setup.ML" begin(*>*)
 
 text {*
@@ -360,11 +359,12 @@
 (*<*)
 
 text{*the following declaration isn't actually used*}
-consts integer_arity :: "integer_op \<Rightarrow> nat"
 primrec
-"integer_arity (Number n)        = 0"
-"integer_arity UnaryMinus        = 1"
-"integer_arity Plus              = 2"
+  integer_arity :: "integer_op \<Rightarrow> nat"
+where
+  "integer_arity (Number n)        = 0"
+| "integer_arity UnaryMinus        = 1"
+| "integer_arity Plus              = 2"
 
 text{* the rest isn't used: too complicated.  OK for an exercise though.*}