Rem unused opens in Safe (#93)

This commit is contained in:
Patrick Stevens
2020-01-05 15:06:35 +00:00
committed by GitHub
parent 019a9d9a07
commit cbe55c9b56
169 changed files with 0 additions and 960 deletions

View File

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