src/HOL/Nat.thy
changeset 1370 7361ac9b024d
parent 1151 c820b3cc3df0
child 1475 7f5a4cd08209
--- a/src/HOL/Nat.thy	Mon Nov 27 13:44:56 1995 +0100
+++ b/src/HOL/Nat.thy	Wed Nov 29 16:44:59 1995 +0100
@@ -19,8 +19,8 @@
   ind :: term
 
 consts
-  Zero_Rep      :: "ind"
-  Suc_Rep       :: "ind => ind"
+  Zero_Rep      :: ind
+  Suc_Rep       :: ind => ind
 
 rules
   (*the axiom of infinity in 2 parts*)
@@ -43,11 +43,11 @@
 (* abstract constants and syntax *)
 
 consts
-  "0"           :: "nat"                ("0")
-  Suc           :: "nat => nat"
-  nat_case      :: "['a, nat => 'a, nat] => 'a"
+  "0"           :: nat                ("0")
+  Suc           :: nat => nat
+  nat_case      :: ['a, nat => 'a, nat] => 'a
   pred_nat      :: "(nat * nat) set"
-  nat_rec       :: "[nat, 'a, [nat, 'a] => 'a] => 'a"
+  nat_rec       :: [nat, 'a, [nat, 'a] => 'a] => 'a
 
 translations
   "case p of 0 => a | Suc(y) => b" == "nat_case a (%y.b) p"