summaryrefslogtreecommitdiff
path: root/README/Case.agda
diff options
context:
space:
mode:
authorSean Whitton <spwhitton@spwhitton.name>2018-11-23 17:29:18 -0700
committerSean Whitton <spwhitton@spwhitton.name>2018-11-23 17:29:18 -0700
commita19b25a865b2000bbd3acd909f5951a5407c1eec (patch)
treee283a809447d00f63289a918e6fd0f73ee0b8ece /README/Case.agda
parent0b3946998d82e1be6c50e2872e7474db69b5a0dc (diff)
New upstream version 0.17
Diffstat (limited to 'README/Case.agda')
-rw-r--r--README/Case.agda4
1 files changed, 2 insertions, 2 deletions
diff --git a/README/Case.agda b/README/Case.agda
index e42f55a..229acf8 100644
--- a/README/Case.agda
+++ b/README/Case.agda
@@ -22,8 +22,8 @@ pred n = case n of λ
; (suc n) → n
}
-from-just : ∀ {a} {A : Set a} (x : Maybe A) → From-just A x
-from-just x = case x return From-just _ of λ
+from-just : ∀ {a} {A : Set a} (x : Maybe A) → From-just x
+from-just x = case x return From-just of λ
{ (just x) → x
; nothing → _
}