Skip to content

Commit 5346ec9

Browse files
committed
refactor: resolve merge conflict following agda#2793
1 parent ddd2669 commit 5346ec9

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Data/Fin/Properties.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -1021,11 +1021,11 @@ module _ {P : Pred (Fin (suc n)) p} where
10211021

10221022
any? : {P : Pred (Fin n) p} Decidable P Dec (∃ P)
10231023
any? {zero} P? = no λ{ (() , _) }
1024-
any? {suc _} P? = Dec.map ⊎⇔∃ (P? zero ⊎-dec any? (P? ∘ suc))
1024+
any? {suc _} P? = Dec.map ⊎⇔∃ (P? zero ⊎? any? (P? ∘ suc))
10251025

10261026
all? : {P : Pred (Fin n) p} Decidable P Dec ( i P i)
10271027
all? {zero} P? = yes λ()
1028-
all? {suc _} P? = Dec.map ∀-cons-⇔ (P? zero ×-dec all? (P? ∘ suc))
1028+
all? {suc _} P? = Dec.map ∀-cons-⇔ (P? zero ×? all? (P? ∘ suc))
10291029

10301030
private
10311031
-- A nice computational property of `all?`:
@@ -1076,7 +1076,7 @@ decFinSubset {suc _} {P = P} {Q = Q} Q? P? = dec[Q⊆P]
10761076
dec[Q⊆P] : Dec (Q ⊆ P)
10771077
dec[Q⊆P] with Q? zero
10781078
... | no ¬q₀ = map′ (cons (contradiction′ ¬q₀)) Q⊆P⇒Q⊆ₛP ih
1079-
... | yes q₀ = map′ (uncurry (cons ∘ const)) < _$ q₀ , Q⊆P⇒Q⊆ₛP > (P? q₀ ×-dec ih)
1079+
... | yes q₀ = map′ (uncurry (cons ∘ const)) < _$ q₀ , Q⊆P⇒Q⊆ₛP > (P? q₀ ×? ih)
10801080

10811081
------------------------------------------------------------------------
10821082
-- Properties of functions to and from Fin

0 commit comments

Comments
 (0)