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.Binary.Sublist.DecSetoid.Solver.html below:

Data.List.Relation.Binary.Sublist.DecSetoid.Solver

Data.List.Relation.Binary.Sublist.DecSetoid.Solver
------------------------------------------------------------------------
-- The Agda standard library
--
-- A solver for proving that one list is a sublist of the other.
------------------------------------------------------------------------

{-# OPTIONS --cubical-compatible --safe #-}

open import Relation.Binary.Bundles using (DecSetoid)

module Data.List.Relation.Binary.Sublist.DecSetoid.Solver {c } (S : DecSetoid c ) where

open DecSetoid S

open import Data.List.Relation.Binary.Sublist.Heterogeneous.Solver _≈_ refl _≟_
  using (Item; module Item; TList; module TList; prove) public

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