Skip to content

Commit 256a505

Browse files
committed
chnage to public re-export of Relation.Nullary.Decidable.Core.decToMaybe
1 parent ab16308 commit 256a505

File tree

3 files changed

+9
-6
lines changed

3 files changed

+9
-6
lines changed

CHANGELOG.md

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -744,7 +744,7 @@ Additions to existing modules
744744
recompute : Reflects A b → Recomputable A
745745
recompute-constant : (r : Reflects A b) (p q : A) → recompute r p ≡ recompute r q
746746
```
747-
747+
748748
* Added new definitions in `Relation.Unary`
749749
```
750750
Stable : Pred A ℓ → Set _

src/Data/Maybe/Base.agda

Lines changed: 7 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -16,7 +16,7 @@ open import Data.Unit.Base using (⊤)
1616
open import Data.These.Base using (These; this; that; these)
1717
open import Data.Product.Base as Prod using (_×_; _,_)
1818
open import Function.Base using (_∘_; id; const)
19-
import Relation.Nullary.Decidable.Core
19+
import Relation.Nullary.Decidable.Core as Dec
2020

2121
private
2222
variable
@@ -134,12 +134,15 @@ thatM : Maybe A → B → These A B
134134
thatM = maybe′ these that
135135

136136
------------------------------------------------------------------------
137-
-- Deprecated
137+
-- DEPRECATED NAMES
138+
------------------------------------------------------------------------
139+
-- Please use the new names as continuing support for the old names is
140+
-- not guaranteed.
138141

139142
-- Version 2.1
140-
-- decToMaybe
143+
-- decToMaybe #2330/2336
141144

142-
decToMaybe = Relation.Nullary.Decidable.Core.decToMaybe
145+
open Dec public using (decToMaybe)
143146
{-# WARNING_ON_USAGE decToMaybe
144147
"Warning: decToMaybe was deprecated in v2.1.
145148
Please use Relation.Nullary.Decidable.Core.decToMaybe instead."

src/Relation/Nullary/Decidable/Core.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,7 @@
1111

1212
module Relation.Nullary.Decidable.Core where
1313

14-
-- decToMaybe was intended to be deprecated in v2.1 #2330/#2336
14+
-- decToMaybe was deprecated in v2.1 #2330/#2336
1515
-- this can go through `Data.Maybe.Base` once that deprecation is fully done.
1616
open import Agda.Builtin.Maybe using (Maybe; just; nothing)
1717

0 commit comments

Comments
 (0)