-
Notifications
You must be signed in to change notification settings - Fork 257
Closed
Description
I saw that in Relation.Binary.Core
is suggested (without expressing it formally) that the containment _⊆_
can be viewed as a synonym of the implication _⇒_
agda-stdlib/src/Relation/Binary/Core.agda
Lines 43 to 46 in 99367e2
-- Implication/containment - could also be written _⊆_. | |
_⇒_ : REL A B ℓ₁ → REL A B ℓ₂ → Set _ | |
P ⇒ Q = ∀ {x y} → P x y → Q x y |
Then in Data.List.Relation.Binary.Sublist.Setoid
the symbol of containment _⊆_
is used to express containment restricted to Lists.
agda-stdlib/src/Data/List/Relation/Binary/Sublist/Setoid.agda
Lines 40 to 41 in 99367e2
_⊆_ : Rel (List A) (c ⊔ ℓ) | |
_⊆_ = Heterogeneous.Sublist _≈_ |
Should not _⊆_
be reserved to express general containment and then notate the specific containments in another way, eg, _⊆ₗᵢₛₜ_
?