File tree 3 files changed +18
-3
lines changed
3 files changed +18
-3
lines changed Original file line number Diff line number Diff line change @@ -49,6 +49,8 @@ idris2docs_venv
49
49
. \# *
50
50
# VS Code
51
51
.vscode /*
52
+ # JetBrains IDEs
53
+ .idea /
52
54
53
55
# macOS
54
56
.DS_Store
Original file line number Diff line number Diff line change @@ -294,6 +294,8 @@ This CHANGELOG describes the merged but unreleased changes. Please see [CHANGELO
294
294
295
295
* Added ` System.Concurrency.getThreadId ` for the chez backend.
296
296
297
+ * ` unrestricted ` , for unpacking a ` !* a ` , now uses its argument once
298
+
297
299
#### Contrib
298
300
299
301
* ` Data.Vect.Views.Extra ` was moved from ` contrib ` to ` base ` .
Original file line number Diff line number Diff line change @@ -21,6 +21,17 @@ public export
21
21
export prefix 5 !*
22
22
||| Prefix notation for the linear unrestricted modality
23
23
public export
24
- record (!* ) (a : Type ) where
25
- constructor MkBang
26
- unrestricted : a
24
+ data (!* ) : Type -> Type where
25
+ MkBang : a -> !* a
26
+
27
+ ||| Unpack an unrestricted value in a linear context
28
+ public export
29
+ unrestricted : !* a -@ a
30
+ unrestricted (MkBang unr) = unr
31
+
32
+ ||| Unpack an unrestricted value in a linear context
33
+ |||
34
+ ||| A postfix alias for function unrestricted.
35
+ public export
36
+ (. unrestricted) : !* a - @ a
37
+ (. unrestricted) = unrestricted
You can’t perform that action at this time.
0 commit comments