File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed
src/Data/Fin/Permutation/Transposition Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -16,7 +16,7 @@ import Data.Fin.Permutation.Components as PC
16
16
open import Data.List as L using (List; []; _∷_; _++_; map)
17
17
import Data.List.Properties as L
18
18
open import Data.Nat.Base using (ℕ; suc; zero)
19
- open import Data.Product using (Σ-syntax; ∃-syntax ; _×_; _,_)
19
+ open import Data.Product using (∃₂ ; _×_; _,_)
20
20
open import Function using (_∘_)
21
21
open import Relation.Binary.PropositionalEquality
22
22
using (_≡_; _≢_; refl; sym; trans; cong; module ≡-Reasoning )
@@ -36,7 +36,7 @@ private
36
36
-- leaving the rest in place).
37
37
38
38
TranspositionList : ℕ → Set
39
- TranspositionList n = List (Σ[ i ∈ Fin n ] ∃[ j ] i ≢ j)
39
+ TranspositionList n = List (∃₂ λ (i j : Fin n) → i ≢ j)
40
40
41
41
------------------------------------------------------------------------
42
42
-- Operations on transposition lists
You can’t perform that action at this time.
0 commit comments