src/FOL/ex/Nat.thy
changeset 41310 65631ca437c9
parent 31974 e81979a703a4
child 41779 a68f503805ed
--- a/src/FOL/ex/Nat.thy	Mon Dec 20 15:24:25 2010 +0100
+++ b/src/FOL/ex/Nat.thy	Mon Dec 20 16:44:33 2010 +0100
@@ -13,7 +13,7 @@
 arities nat :: "term"
 
 consts
-  0 :: nat    ("0")
+  Zero :: nat    ("0")
   Suc :: "nat => nat"
   rec :: "[nat, 'a, [nat, 'a] => 'a] => 'a"
   add :: "[nat, nat] => nat"    (infixl "+" 60)