Skip to content

Commit 6a51764

Browse files
UlfNorellgallais
authored andcommitted
Add implicit arguments required after fix of agda/agda#4174
1 parent 1595db8 commit 6a51764

File tree

2 files changed

+3
-3
lines changed

2 files changed

+3
-3
lines changed

src/Data/List/Relation/Binary/Permutation/Propositional/Properties.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -112,7 +112,7 @@ module _ {a} {A : Set a} where
112112
x ∷ v ∷ xs ++ ys <<⟨ refl ⟩
113113
v ∷ x ∷ xs ++ ys ∎
114114

115-
drop-mid-≡ : {x} ws xs {ys} {zs}
115+
drop-mid-≡ : {x : A} ws xs {ys} {zs}
116116
ws ++ [ x ] ++ ys ≡ xs ++ [ x ] ++ zs
117117
ws ++ ys ↭ xs ++ zs
118118
drop-mid-≡ [] [] eq with cong tail eq
@@ -291,7 +291,7 @@ module _ {a} {A : Set a} where
291291
... | res rewrite ↭-sym-involutive p = res
292292

293293
∼bag⇒↭ : _∼[ bag ]_ ⇒ _↭_
294-
∼bag⇒↭ {[]} eq with empty-unique (Inv.sym eq)
294+
∼bag⇒↭ {[]} eq with empty-unique {A = A} (Inv.sym eq)
295295
... | refl = refl
296296
∼bag⇒↭ {x ∷ xs} eq with ∈-∃++ (to ⟨$⟩ (here ≡.refl))
297297
where open Inv.Inverse (eq {x})

src/Data/List/Relation/Unary/Any/Properties.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -230,7 +230,7 @@ module _ {P : Pred A p} {Q : Pred B q} where
230230
| lose∘find q
231231
= refl
232232

233-
to∘from : pq Any-×⁺ (Any-×⁻ pq) ≡ pq
233+
to∘from : pq Any-×⁺ {xs} (Any-×⁻ pq) ≡ pq
234234
to∘from pq
235235
with find pq
236236
| (λ (f : (proj₁ (find pq) ≡_) ⋐ _) map∘find pq {f})

0 commit comments

Comments
 (0)