src/HOL/TLA/Memory/MIParameters.thy
changeset 11703 6e5de8d4290a
parent 5184 9b8547a9496a
child 17309 c43ed29bd197
--- a/src/HOL/TLA/Memory/MIParameters.thy	Fri Oct 05 23:58:17 2001 +0200
+++ b/src/HOL/TLA/Memory/MIParameters.thy	Fri Oct 05 23:58:52 2001 +0200
@@ -9,9 +9,8 @@
     RPC-Memory example: Parameters of the memory implementation.
 *)
 
-MIParameters = Datatype +
+MIParameters = Main +
 
 datatype  histState  =  histA | histB
 
 end
-