src/HOL/Induct/Com.thy
changeset 5184 9b8547a9496a
parent 5102 8c782c25a11e
child 10759 994877ee68cb
--- a/src/HOL/Induct/Com.thy	Fri Jul 24 13:03:20 1998 +0200
+++ b/src/HOL/Induct/Com.thy	Fri Jul 24 13:19:38 1998 +0200
@@ -6,7 +6,7 @@
 Example of Mutual Induction via Iteratived Inductive Definitions: Commands
 *)
 
-Com = Arith + Inductive +
+Com = Datatype +
 
 types loc
       state = "loc => nat"