Move Functions (#119)

This commit is contained in:
Patrick Stevens
2020-04-18 17:47:27 +01:00
committed by GitHub
parent 84a146f72c
commit 1831ef49c4
112 changed files with 203 additions and 193 deletions

View File

@@ -1,6 +1,6 @@
{-# OPTIONS --safe --warning=error --without-K #-}
open import Functions
open import Functions.Definition
open import Agda.Primitive using (Level; lzero; lsuc; _⊔_)
open import LogicalFormulae
open import Setoids.Subset