File tree Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Expand file tree Collapse file tree 1 file changed +2
-2
lines changed Original file line number Diff line number Diff line change @@ -25,7 +25,7 @@ open import Data.List.Membership.Propositional.Properties using (∈-∃++)
25
25
open import Data.List.Relation.Unary.All as All using (All; []; _∷_)
26
26
open import Data.List.Relation.Unary.Any using (here; there)
27
27
open import Data.List.Relation.Binary.Permutation.Propositional
28
- using (_↭_; prep; swap; ↭-reflexive; ↭-refl; ↭-trans; refl ; module PermutationReasoning )
28
+ using (_↭_; ↭-reflexive; ↭-refl; ↭-trans; module PermutationReasoning )
29
29
open import Data.List.Relation.Binary.Permutation.Propositional.Properties
30
30
using (All-resp-↭; shift)
31
31
open import Data.Sum.Base using (inj₁; inj₂)
@@ -147,7 +147,7 @@ factorisationHasAllPrimeFactors {a ∷ as} {p} pPrime p∣aΠas (aPrime ∷ asPr
147
147
148
148
private
149
149
factorisationUnique′ : (as bs : List ℕ) → product as ≡ product bs → All Prime as → All Prime bs → as ↭ bs
150
- factorisationUnique′ [] [] Πas≡Πbs asPrime bsPrime = refl
150
+ factorisationUnique′ [] [] Πas≡Πbs asPrime bsPrime = ↭- refl
151
151
factorisationUnique′ [] (b@(2+ _) ∷ bs) Πas≡Πbs prime[as] (_ ∷ prime[bs]) =
152
152
contradiction Πas≡Πbs (<⇒≢ Πas<Πbs)
153
153
where
You can’t perform that action at this time.
0 commit comments