File tree Expand file tree Collapse file tree 2 files changed +3
-3
lines changed
Binary/Permutation/Propositional Expand file tree Collapse file tree 2 files changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -112,7 +112,7 @@ module _ {a} {A : Set a} where
112
112
x ∷ v ∷ xs ++ ys <<⟨ refl ⟩
113
113
v ∷ x ∷ xs ++ ys ∎
114
114
115
- drop-mid-≡ : ∀ {x} ws xs {ys} {zs} →
115
+ drop-mid-≡ : ∀ {x : A } ws xs {ys} {zs} →
116
116
ws ++ [ x ] ++ ys ≡ xs ++ [ x ] ++ zs →
117
117
ws ++ ys ↭ xs ++ zs
118
118
drop-mid-≡ [] [] eq with cong tail eq
@@ -291,7 +291,7 @@ module _ {a} {A : Set a} where
291
291
... | res rewrite ↭-sym-involutive p = res
292
292
293
293
∼bag⇒↭ : _∼[ bag ]_ ⇒ _↭_
294
- ∼bag⇒↭ {[]} eq with empty-unique (Inv.sym eq)
294
+ ∼bag⇒↭ {[]} eq with empty-unique {A = A} (Inv.sym eq)
295
295
... | refl = refl
296
296
∼bag⇒↭ {x ∷ xs} eq with ∈-∃++ (to ⟨$⟩ (here ≡.refl))
297
297
where open Inv.Inverse (eq {x})
Original file line number Diff line number Diff line change @@ -230,7 +230,7 @@ module _ {P : Pred A p} {Q : Pred B q} where
230
230
| lose∘find q
231
231
= refl
232
232
233
- to∘from : ∀ pq → Any-×⁺ (Any-×⁻ pq) ≡ pq
233
+ to∘from : ∀ pq → Any-×⁺ {xs} (Any-×⁻ pq) ≡ pq
234
234
to∘from pq
235
235
with find pq
236
236
| (λ (f : (proj₁ (find pq) ≡_) ⋐ _) → map∘find pq {f})
You can’t perform that action at this time.
0 commit comments