Skip to content

Commit 84c9420

Browse files
committed
refactor: knock-ons
1 parent 5619f17 commit 84c9420

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Data/Fin/Permutation.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ open import Data.Bool.Base using (true; false)
1212
open import Data.Fin.Base using (Fin; suc; opposite; punchIn; punchOut)
1313
open import Data.Fin.Patterns using (0F)
1414
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)
1616
import Data.Fin.Permutation.Components as PC
1717
open import Data.Nat.Base using (ℕ; suc; zero)
1818
open import Data.Product.Base using (_,_; proj₂)
@@ -197,7 +197,7 @@ insert {m} {n} i j π = permutation to from inverseˡ′ inverseʳ′
197197

198198
inverseʳ′ : StrictlyInverseʳ _≡_ to from
199199
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
201201
... | no i≢k
202202
with j≢punchInⱼπʳpunchOuti≢k punchInᵢ≢i j (π ⟨$⟩ʳ punchOut i≢k) ∘ sym
203203
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ʳ′
210210

211211
inverseˡ′ : StrictlyInverseˡ _≡_ to from
212212
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
214214
... | no j≢k
215215
with i≢punchInᵢπˡpunchOutj≢k punchInᵢ≢i i (π ⟨$⟩ˡ punchOut j≢k) ∘ sym
216216
rewrite dec-no (i ≟ punchIn i (π ⟨$⟩ˡ punchOut j≢k)) i≢punchInᵢπˡpunchOutj≢k

0 commit comments

Comments
 (0)