Reshuffle orders (#91)

This commit is contained in:
Patrick Stevens
2019-12-29 12:11:21 +00:00
committed by GitHub
parent 876396eaaa
commit b6ef9b46f2
57 changed files with 476 additions and 462 deletions

View File

@@ -0,0 +1,14 @@
{-# OPTIONS --safe --warning=error --without-K #-}
open import LogicalFormulae
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import Functions
module Orders.WellFounded.Definition {a b : _} {A : Set a} (_<_ : Rel {a} {b} A) where
data Accessible (x : A) : Set (lsuc a b) where
access : ( y y < x Accessible y) Accessible x
WellFounded : Set (lsuc a b)
WellFounded = x Accessible x