File tree Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Expand file tree Collapse file tree 1 file changed +3
-3
lines changed Original file line number Diff line number Diff line change @@ -1021,11 +1021,11 @@ module _ {P : Pred (Fin (suc n)) p} where
10211021
10221022any? : ∀ {P : Pred (Fin n) p} → Decidable P → Dec (∃ P)
10231023any? {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
10261026all? : ∀ {P : Pred (Fin n) p} → Decidable P → Dec (∀ i → P i)
10271027all? {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
10301030private
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
You can’t perform that action at this time.
0 commit comments