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.Maybe.html below:

Data.Maybe

Data.Maybe
------------------------------------------------------------------------
-- The Agda standard library
--
-- The Maybe type
------------------------------------------------------------------------

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

module Data.Maybe where

open import Data.Empty using ()
open import Data.Unit.Base using ()
open import Data.Bool.Base using (T)
open import Data.Maybe.Relation.Unary.All using (All)
open import Data.Maybe.Relation.Unary.Any using (Any; just)
open import Level using (Level)

private
  variable
    a : Level
    A : Set a

------------------------------------------------------------------------
-- The base type and some operations

open import Data.Maybe.Base public

------------------------------------------------------------------------
-- Using Any and All to define Is-just and Is-nothing

Is-just : Maybe A  Set _
Is-just = Any  _  )

Is-nothing : Maybe A  Set _
Is-nothing = All  _  )

to-witness :  {m : Maybe A}  Is-just m  A
to-witness (just {x = p} _) = p

to-witness-T :  (m : Maybe A)  T (is-just m)  A
to-witness-T (just p) _  = p

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