We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
import
1 parent df74251 commit d8f1e47Copy full SHA for d8f1e47
src/Relation/Nullary/Reflects.agda
@@ -14,7 +14,7 @@ open import Data.Bool.Base
14
open import Data.Sum.Base using (_⊎_; inj₁; inj₂)
15
open import Data.Product.Base using (_×_; _,_; proj₁; proj₂)
16
open import Level using (Level)
17
-open import Function.Base using (_$_; _∘_; const; id; flip)
+open import Function.Base using (_$_; _∘_; const; id)
18
open import Relation.Nullary.Negation.Core using (¬_; weak-contradiction; _¬-⊎_)
19
open import Relation.Nullary.Recomputable using (Recomputable)
20
0 commit comments