Skip to content

Commit 1f1eaf5

Browse files
committed
rename Irrelevant′ as Recomputable
1 parent 6daa0fb commit 1f1eaf5

File tree

3 files changed

+9
-9
lines changed

3 files changed

+9
-9
lines changed

CHANGELOG.md

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -308,10 +308,10 @@ Other minor additions
308308
≢-sym : Symmetric _≢_
309309
```
310310

311-
* Defined another notion of irrelevance (reconstructibility) for binary relations:
311+
* Defined a notion of recomputability for binary relations:
312312
```agda
313-
Irrelevant′ : REL A B ℓ → Set _
314-
Irrelevant′ _~_ = ∀ {x y} → .(x ~ y) → x ~ y
313+
Recomputable : REL A B ℓ → Set _
314+
Recomputable _~_ = ∀ {x y} → .(x ~ y) → x ~ y
315315
316-
dec⟶irrel′ : Decidable R → Irrelevant′ R
316+
dec⟶recomput : Decidable R → Recomputable R
317317
```

src/Relation/Binary/Consequences.agda

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -167,5 +167,5 @@ module _ {P : REL A B ℓ₁} {Q : REL B A ℓ₂} where
167167

168168
module _ {r} {R : REL A B r} where
169169

170-
dec⟶irrel′ : Decidable R Irrelevant′ R
171-
dec⟶irrel′ dec {a} {b} = recompute $ dec a b
170+
dec⟶recomput : Decidable R Recomputable R
171+
dec⟶recomput dec {a} {b} = recompute $ dec a b

src/Relation/Binary/Core.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -217,11 +217,11 @@ WeaklyDecidable _∼_ = ∀ x y → Maybe (x ∼ y)
217217
Irrelevant : REL A B ℓ Set _
218218
Irrelevant _∼_ = {x y} (a b : x ∼ y) a ≡ b
219219

220-
-- Another irrelevancy - we can rebuild a relevant proof given an
220+
-- Recomputability - we can rebuild a relevant proof given an
221221
-- irrelevant one.
222222

223-
Irrelevant′ : REL A B ℓ Set _
224-
Irrelevant′ _∼_ = {x y} .(x ∼ y) x ∼ y
223+
Recomputable : REL A B ℓ Set _
224+
Recomputable _∼_ = {x y} .(x ∼ y) x ∼ y
225225

226226
-- Universal - all pairs of elements are related
227227

0 commit comments

Comments
 (0)