We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 617bd62 commit 1f67befCopy full SHA for 1f67bef
src/Data/Fin/Properties.agda
@@ -47,8 +47,7 @@ open import Relation.Binary.PropositionalEquality.Properties as ≡
47
open import Relation.Nullary.Decidable as Dec
48
using (Dec; _because_; yes; no; _×-dec_; _⊎-dec_; map′)
49
open import Relation.Nullary.Negation.Core using (¬_; contradiction)
50
-open import Relation.Nullary.Recomputable using (¬-recompute)
51
-open import Relation.Nullary.Reflects using (Reflects; invert)
+open import Relation.Nullary.Reflects using (invert)
52
open import Relation.Unary as U
53
using (U; Pred; Decidable; _⊆_; Satisfiable; Universal)
54
open import Relation.Unary.Properties using (U?)
0 commit comments