Skip to content

Commit

Permalink
refactor: cosmetic, tighten imports
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna committed Jan 17, 2025
1 parent 56d0a74 commit e37fe01
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions src/Data/Nat/Primality/Factorisation.agda
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,7 @@ open import Data.List.Membership.Propositional.Properties using (∈-∃++)
open import Data.List.Relation.Unary.All as All using (All; []; _∷_)
open import Data.List.Relation.Unary.Any using (here; there)
open import Data.List.Relation.Binary.Permutation.Propositional
using (_↭_; prep; swap; ↭-reflexive; ↭-refl; ↭-trans; refl; module PermutationReasoning)
using (_↭_; ↭-reflexive; ↭-refl; ↭-trans; module PermutationReasoning)
open import Data.List.Relation.Binary.Permutation.Propositional.Properties
using (All-resp-↭; shift)
open import Data.Sum.Base using (inj₁; inj₂)
Expand Down Expand Up @@ -147,7 +147,7 @@ factorisationHasAllPrimeFactors {a ∷ as} {p} pPrime p∣aΠas (aPrime ∷ asPr

private
factorisationUnique′ : (as bs : List ℕ) product as ≡ product bs All Prime as All Prime bs as ↭ bs
factorisationUnique′ [] [] Πas≡Πbs asPrime bsPrime = refl
factorisationUnique′ [] [] Πas≡Πbs asPrime bsPrime = ↭-refl
factorisationUnique′ [] (b@(2+ _) ∷ bs) Πas≡Πbs prime[as] (_ ∷ prime[bs]) =
contradiction Πas≡Πbs (<⇒≢ Πas<Πbs)
where
Expand Down

0 comments on commit e37fe01

Please sign in to comment.