src/FOL/ex/Nat_Class.thy
changeset 44605 4877c4e184e5
parent 29753 a9fc00f1b8f0
child 60770 240563fbf41d
--- a/src/FOL/ex/Nat_Class.thy	Tue Aug 30 17:53:03 2011 +0200
+++ b/src/FOL/ex/Nat_Class.thy	Tue Aug 30 18:12:48 2011 +0200
@@ -26,9 +26,8 @@
     and rec_Suc: "rec(Suc(m), a, f) = f(m, rec(m, a, f))"
 begin
 
-definition
-  add :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "+" 60) where
-  "m + n = rec(m, n, \<lambda>x y. Suc(y))"
+definition add :: "'a \<Rightarrow> 'a \<Rightarrow> 'a"  (infixl "+" 60)
+  where "m + n = rec(m, n, \<lambda>x y. Suc(y))"
 
 lemma Suc_n_not_n: "Suc(k) \<noteq> (k::'a)"
   apply (rule_tac n = k in induct)