diff -r 3395fe5e3893 -r a095acd4cfbf src/HOL/UNITY/Follows.thy --- a/src/HOL/UNITY/Follows.thy Tue Jul 05 10:26:23 2016 +0200 +++ b/src/HOL/UNITY/Follows.thy Tue Jul 05 13:05:04 2016 +0200 @@ -175,19 +175,7 @@ subsection\Multiset union properties (with the multiset ordering)\ -(*TODO: remove when multiset is of sort ord again*) -instantiation multiset :: (order) ordered_ab_semigroup_add -begin -definition less_multiset :: "'a::order multiset \ 'a multiset \ bool" where - "M' < M \ M' #\# M" - -definition less_eq_multiset :: "'a multiset \ 'a multiset \ bool" where - "(M'::'a multiset) \ M \ M' #\# M" - -instance - by standard (auto simp add: less_eq_multiset_def less_multiset_def multiset_order.less_le_not_le add.commute multiset_order.add_right_mono) -end lemma increasing_union: "[| F \ increasing f; F \ increasing g |]