src/HOL/ex/Fundefs.thy
changeset 22492 43545e640877
parent 22166 0a50d4db234a
child 22618 e40957ccf0e9
--- a/src/HOL/ex/Fundefs.thy	Wed Mar 21 13:58:36 2007 +0100
+++ b/src/HOL/ex/Fundefs.thy	Wed Mar 21 16:06:15 2007 +0100
@@ -114,9 +114,9 @@
 function gcd3 :: "nat \<Rightarrow> nat \<Rightarrow> nat"
 where
   "gcd3 x 0 = x"
-  "gcd3 0 y = y"
-  "x < y \<Longrightarrow> gcd3 (Suc x) (Suc y) = gcd3 (Suc x) (y - x)"
-  "\<not> x < y \<Longrightarrow> gcd3 (Suc x) (Suc y) = gcd3 (x - y) (Suc y)"
+| "gcd3 0 y = y"
+| "x < y \<Longrightarrow> gcd3 (Suc x) (Suc y) = gcd3 (Suc x) (y - x)"
+| "\<not> x < y \<Longrightarrow> gcd3 (Suc x) (Suc y) = gcd3 (x - y) (Suc y)"
   apply (case_tac x, case_tac a, auto)
   apply (case_tac ba, auto)
   done
@@ -131,7 +131,7 @@
 function ev :: "nat \<Rightarrow> bool"
 where
   "ev (2 * n) = True"
-  "ev (2 * n + 1) = False"
+| "ev (2 * n + 1) = False"
 proof -  -- {* completeness is more difficult here \dots *}
   fix P :: bool
     and x :: nat