File tree Expand file tree Collapse file tree 2 files changed +10
-0
lines changed
src/Data/List/Relation/Unary/First Expand file tree Collapse file tree 2 files changed +10
-0
lines changed Original file line number Diff line number Diff line change @@ -448,6 +448,11 @@ Other minor additions
448448 all-upTo : All (_< n) (upTo n)
449449 ```
450450
451+ * Added new proof in ` Data.List.Relation.Unary.First.Properties ` :
452+ ``` agda
453+ cofirst? : Decidable P → Decidable (First (∁ P) P)
454+ ```
455+
451456* Added new operations in ` Data.List.Relation.Unary.Linked ` :
452457 ``` agda
453458 head′ : Linked R (x ∷ xs) → Connected R (just x) (head xs)
Original file line number Diff line number Diff line change @@ -85,6 +85,11 @@ module _ {a p} {A : Set a} {P : Pred A p} where
8585 $ Sum.map₂ (All⇒¬First contradiction)
8686 $ first (Sum.fromDec ∘ P?) xs
8787
88+ cofirst? : Decidable P → Decidable (First (∁ P) P)
89+ cofirst? P? xs = Sum.toDec
90+ $ Sum.map₂ (All⇒¬First id)
91+ $ first (Sum.swap ∘ Sum.fromDec ∘ P?) xs
92+
8893------------------------------------------------------------------------
8994-- Conversion to Any
9095
You can’t perform that action at this time.
0 commit comments