We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
_⟨⟩
1 parent 13db471 commit 306d2eaCopy full SHA for 306d2ea
lib/base/Haskell/Extra/Refinement.agda
@@ -7,17 +7,14 @@ private variable
7
ℓ ℓ′ : Level
8
9
record ∃ (a : Type ℓ) (@0 P : a → Type ℓ′) : Type (ℓ ⊔ ℓ′) where
10
- constructor _⟨_⟩
+ constructor _⟨⟩
11
field
12
value : a
13
- @0 proof : P value
+ @0 {{proof}} : P value
14
open ∃ public
15
{-# COMPILE AGDA2HS ∃ unboxed #-}
16
17
-_⟨⟩ : {@0 P : a → Type ℓ} (x : a) → @0 {{P x}} → ∃ a P
18
-(x ⟨⟩) {{p}} = x ⟨ p ⟩
19
-
20
-{-# COMPILE AGDA2HS _⟨⟩ inline #-}
+pattern _⟨_⟩ x p = (x ⟨⟩) {{p}}
21
22
mapRefine : {@0 P Q : a → Type ℓ} (@0 f : ∀ {x} → P x → Q x) → ∃ a P → ∃ a Q
23
mapRefine f (x ⟨ p ⟩) = x ⟨ f p ⟩
0 commit comments