Closed
Description
I'm using Agda version 2.6.4 and standard-library-2.0
In the fixing a working code in Agda 2.6.3 and standard-library, (simialar one with Data.Fin.Permutation.remove
)
p← : Fin n → Fin n
p← x with perm ⟨$⟩ˡ (suc x) in eq
p← x | zero = ⊥-elim ( sh2 perm p0=0 {x} eq )
p← x | suc t = t
p01 : (x : Fin n) → ?
p01 x with perm ⟨$⟩ˡ (suc x)
... | t = ?
bad1 : (x : Fin n) → Fin (suc n)
bad1 x = perm ⟨$⟩ˡ (suc x)
bad : (x : Fin n) → p← x ≡ ?
bad with bad1 x
... | t = ?
This gives me ...
/Users/kono/src/galois/src/pm.agda:60,4-15
Function.Bundles.Inverse.from perm (suc x) != w of type Fin (suc n)
when checking that the type
{n : ℕ} (perm : Permutation (suc n) (suc n)) (x : Fin n)
(w : Fin (suc n))
(p0=0 : Function.Bundles.Inverse.from perm zero ≡ zero) →
(p← perm p0=0 x | w | refl) ≡
?2 (perm = perm) (p0=0 = p0=0) (x = x)
of the generated with function is well-formed