File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -12,7 +12,7 @@ open import Data.Bool.Base using (true; false)
12
12
open import Data.Fin.Base using (Fin; suc; opposite; punchIn; punchOut)
13
13
open import Data.Fin.Patterns using (0F)
14
14
open import Data.Fin.Properties using (punchInᵢ≢i; punchOut-punchIn;
15
- punchOut-cong; punchOut-cong′; punchIn-punchOut; _≟_; ¬Fin0)
15
+ punchOut-cong; punchOut-cong′; punchIn-punchOut; _≟_; ¬Fin0; ≟-diag-refl )
16
16
import Data.Fin.Permutation.Components as PC
17
17
open import Data.Nat.Base using (ℕ; suc; zero)
18
18
open import Data.Product.Base using (_,_; proj₂)
@@ -197,7 +197,7 @@ insert {m} {n} i j π = permutation to from inverseˡ′ inverseʳ′
197
197
198
198
inverseʳ′ : StrictlyInverseʳ _≡_ to from
199
199
inverseʳ′ k with i ≟ k
200
- ... | yes i≡k rewrite proj₂ (dec-yes (j ≟ j) refl) = i≡k
200
+ ... | yes i≡k rewrite ≟-diag-refl j = i≡k
201
201
... | no i≢k
202
202
with j≢punchInⱼπʳpunchOuti≢k ← punchInᵢ≢i j (π ⟨$⟩ʳ punchOut i≢k) ∘ sym
203
203
rewrite dec-no (j ≟ punchIn j (π ⟨$⟩ʳ punchOut i≢k)) j≢punchInⱼπʳpunchOuti≢k
@@ -210,7 +210,7 @@ insert {m} {n} i j π = permutation to from inverseˡ′ inverseʳ′
210
210
211
211
inverseˡ′ : StrictlyInverseˡ _≡_ to from
212
212
inverseˡ′ k with j ≟ k
213
- ... | yes j≡k rewrite proj₂ (dec-yes (i ≟ i) refl) = j≡k
213
+ ... | yes j≡k rewrite ≟-diag-refl i = j≡k
214
214
... | no j≢k
215
215
with i≢punchInᵢπˡpunchOutj≢k ← punchInᵢ≢i i (π ⟨$⟩ˡ punchOut j≢k) ∘ sym
216
216
rewrite dec-no (i ≟ punchIn i (π ⟨$⟩ˡ punchOut j≢k)) i≢punchInᵢπˡpunchOutj≢k
You can’t perform that action at this time.
0 commit comments