A RetroSearch Logo

Home - News ( United States | United Kingdom | Italy | Germany ) - Football scores

Search Query:

Showing content from https://agda.github.io/agda-stdlib/master/Data.List.Relation.Ternary.Appending.Setoid.html below:

Data.List.Relation.Ternary.Appending.Setoid

Data.List.Relation.Ternary.Appending.Setoid
------------------------------------------------------------------------
-- The Agda standard library
--
-- Appending of lists using setoid equality
------------------------------------------------------------------------

{-# 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)

------------------------------------------------------------------------
-- Definition

Appending : List A  List A  List A  Set (c  )
Appending = General.Appending _≈_ _≈_

------------------------------------------------------------------------
-- Re-export the basic combinators

open General {A = A} {A} {A} public
  hiding (Appending)

RetroSearch is an open source project built by @garambo | Open a GitHub Issue

Search and Browse the WWW like it's 1997 | Search results from DuckDuckGo

HTML: 3.2 | Encoding: UTF-8 | Version: 0.7.4