src/HOL/Relation.thy
changeset 31011 506e57123cd1
parent 30198 922f944f03b2
child 32235 8f9b8d14fc9f
--- a/src/HOL/Relation.thy	Tue Apr 28 13:34:46 2009 +0200
+++ b/src/HOL/Relation.thy	Tue Apr 28 13:34:48 2009 +0200
@@ -6,7 +6,8 @@
 header {* Relations *}
 
 theory Relation
-imports Datatype Finite_Set
+imports Finite_Set Datatype
+  (*FIXME order is important, otherwise merge problem for canonical interpretation of class monoid_mult wrt. power!*)
 begin
 
 subsection {* Definitions *}