File tree Expand file tree Collapse file tree 3 files changed +9
-9
lines changed Expand file tree Collapse file tree 3 files changed +9
-9
lines changed Original file line number Diff line number Diff line change @@ -308,10 +308,10 @@ Other minor additions
308
308
≢-sym : Symmetric _≢_
309
309
```
310
310
311
- * Defined another notion of irrelevance (reconstructibility) for binary relations:
311
+ * Defined a notion of recomputability for binary relations:
312
312
``` 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
315
315
316
- dec⟶irrel′ : Decidable R → Irrelevant′ R
316
+ dec⟶recomput : Decidable R → Recomputable R
317
317
```
Original file line number Diff line number Diff line change @@ -167,5 +167,5 @@ module _ {P : REL A B ℓ₁} {Q : REL B A ℓ₂} where
167
167
168
168
module _ {r} {R : REL A B r} where
169
169
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
Original file line number Diff line number Diff line change @@ -217,11 +217,11 @@ WeaklyDecidable _∼_ = ∀ x y → Maybe (x ∼ y)
217
217
Irrelevant : REL A B ℓ → Set _
218
218
Irrelevant _∼_ = ∀ {x y} (a b : x ∼ y) → a ≡ b
219
219
220
- -- Another irrelevancy - we can rebuild a relevant proof given an
220
+ -- Recomputability - we can rebuild a relevant proof given an
221
221
-- irrelevant one.
222
222
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
225
225
226
226
-- Universal - all pairs of elements are related
227
227
You can’t perform that action at this time.
0 commit comments