Absorption of sets #
Let M act on α, let A and B be sets in α.
We say that A absorbs B if for sufficiently large a : M, we have B ⊆ a • A.
Formally, "for sufficiently large a : M" means "for all but a bounded set of a".
Traditionally, this definition is formulated for the action of a (semi)normed ring on a module over that ring.
We formulate it in a more general settings for two reasons:
- this way we don't have to depend on metric spaces, normed rings etc;
- some proofs look nicer with this definition than with something like
∃ r : ℝ, ∀ a : R, r ≤ ‖a‖ → B ⊆ a • A.
Implementation notes #
For now, all theorems assume that we deal with (a generalization of) a module over a division ring.
Some lemmas have multiplicative versions for MulDistribMulActions.
They can be added later when someone needs them.
Keywords #
absorbs, absorbent
Alias of Absorbs.empty.
Alias of the forward direction of absorbs_iff_eventually_cobounded_mapsTo.
Alias of the reverse direction of Set.Finite.absorbs_sInter.
Alias of the reverse direction of absorbs_iInter.
Alias of the reverse direction of Set.Finite.absorbs_biInter.
Alias of the forward direction of absorbs_neg_neg.
Alias of the reverse direction of absorbs_neg_neg.