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.Product.Relation.Unary.All.html below:

Data.Product.Relation.Unary.All

Data.Product.Relation.Unary.All
------------------------------------------------------------------------
-- The Agda standard library
--
-- Lifting of two predicates
------------------------------------------------------------------------

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

module Data.Product.Relation.Unary.All where

open import Level using (Level; _⊔_)
open import Data.Product.Base using (_×_; _,_)

private
  variable
    a b p q : Level
    A : Set a
    B : Set b

All : (A  Set p)  (B  Set q)  (A × B  Set (p  q))
All P Q (a , b) = P a × Q b

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