src/HOL/Library/Poly_Mapping.thy
changeset 73655 26a1d66b9077
parent 70045 7b6add80e3a5
child 73932 fd21b4a93043
--- a/src/HOL/Library/Poly_Mapping.thy	Mon May 10 14:28:37 2021 +0200
+++ b/src/HOL/Library/Poly_Mapping.thy	Mon May 10 16:14:34 2021 +0200
@@ -1796,7 +1796,7 @@
 
 lemma keys_frag_extend: "Poly_Mapping.keys(frag_extend f c) \<subseteq> (\<Union>x \<in> Poly_Mapping.keys c. Poly_Mapping.keys(f x))"
   unfolding frag_extend_def
-  by (smt SUP_mono' keys_cmul keys_sum order_trans)
+  using keys_sum by fastforce
 
 lemma frag_expansion: "a = frag_extend frag_of a"
 proof -