moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
(* Title: HOL/ex/Interpretation_with_Defs.thy
Author: Florian Haftmann, TU Muenchen
*)
header {* Interpretation accompanied with mixin definitions. EXPERIMENTAL. *}
theory Interpretation_with_Defs
imports Pure
uses "~~/src/Tools/interpretation_with_defs.ML"
begin
end