Data.List.Relation.Ternary.Appending.Setoid
{-# OPTIONS --cubical-compatible --safe #-}
open import Relation.Binary.Bundles using (Setoid)
module Data.List.Relation.Ternary.Appending.Setoid
{c ℓ} (S : Setoid c ℓ)
where
open import Level using (_⊔_)
open import Data.List.Base as List using (List)
import Data.List.Relation.Ternary.Appending as General
open Setoid S renaming (Carrier to A)
Appending : List A → List A → List A → Set (c ⊔ ℓ)
Appending = General.Appending _≈_ _≈_
open General {A = A} {A} {A} public
hiding (Appending)