type-theory/src/Divergence.agda

16 lines
326 B
Agda
Raw Normal View History

2023-02-23 10:20:35 +00:00
{-# OPTIONS --cubical #-}
module Divergence where
open import Cubical.Core.Everything
open import Cubical.Foundations.Prelude
open import Data.Nat
open import Relation.Binary.Core using (Rel)
open import Relation.Nullary using (¬_)
_≢_ : { : Level} {A : Set } Rel A
x y = ¬ x y
_ : 0 1
_ = ?