------------------------------------------------------------------------
-- The Agda standard library
--
-- Results concerning double negation elimination.
------------------------------------------------------------------------

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

module Axiom.DoubleNegationElimination where

open import Axiom.ExcludedMiddle
open import Level
open import Relation.Nullary.Decidable.Core
  using (decidable-stable; ¬¬-excluded-middle)
open import Relation.Nullary.Negation.Core using (Stable)

private
  variable
     : Level

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

-- The classical statement of double negation elimination says that
-- if a property is not not true then it is true.

DoubleNegationElimination :    Set (suc )
DoubleNegationElimination  = {P : Set }  Stable P

------------------------------------------------------------------------
-- Properties

-- Double negation elimination is equivalent to excluded middle

em⇒dne : ExcludedMiddle   DoubleNegationElimination 
em⇒dne em = decidable-stable em

dne⇒em : DoubleNegationElimination   ExcludedMiddle 
dne⇒em dne = dne ¬¬-excluded-middle