src/HOL/Induct/Com.thy
changeset 5102 8c782c25a11e
parent 4264 5e21f41ccd21
child 5184 9b8547a9496a
--- a/src/HOL/Induct/Com.thy	Tue Jun 30 20:50:34 1998 +0200
+++ b/src/HOL/Induct/Com.thy	Tue Jun 30 20:51:15 1998 +0200
@@ -6,7 +6,7 @@
 Example of Mutual Induction via Iteratived Inductive Definitions: Commands
 *)
 
-Com = Arith +
+Com = Arith + Inductive +
 
 types loc
       state = "loc => nat"