view Paper/src/agda/fresh_test.agda @ 32:4915eaa51ee0 default tip

Add front
author soto <soto@cr.ie.u-ryukyu.ac.jp>
date Thu, 23 Feb 2023 18:39:56 +0900
parents a72446879486
children
line wrap: on
line source

module fresh_test where

open import Data.Nat
open import Data.List.Base
open import Data.List.Fresh
open import Data.List.Relation.Unary.AllPairs as AllPairs using (AllPairs)
open import Data.Product
open import Relation.Nary using (⌊_⌋; fromWitness)

ISortedList : Set
ISortedList = List# ℕ ⌊ _>?_ ⌋

ins : ISortedList
ins = 8 ∷# 4 ∷# 2 ∷# 0 ∷# []