src/HOL/Induct/Comb.thy
changeset 5184 9b8547a9496a
parent 5102 8c782c25a11e
child 9101 b643f4d7b9e9
--- a/src/HOL/Induct/Comb.thy	Fri Jul 24 13:03:20 1998 +0200
+++ b/src/HOL/Induct/Comb.thy	Fri Jul 24 13:19:38 1998 +0200
@@ -13,7 +13,7 @@
 *)
 
 
-Comb = Arith + Inductive +
+Comb = Datatype +
 
 (** Datatype definition of combinators S and K, with infixed application **)
 datatype comb = K