Skip to content

Commit 71362d4

Browse files
committed
Refine some Function.Equality imports
1 parent ef3a22e commit 71362d4

File tree

2 files changed

+8
-1
lines changed

2 files changed

+8
-1
lines changed

src/Function/Equality.agda

+6
Original file line numberDiff line numberDiff line change
@@ -11,6 +11,7 @@
1111
-- `Bijection`. The alternative definitions found in this file will
1212
-- eventually be deprecated.
1313

14+
-- check if modules are actually using Function.Equality and port them
1415
module Function.Equality where
1516

1617
import Function.Base as Fun
@@ -24,6 +25,7 @@ import Relation.Binary.Indexed.Heterogeneous.Construct.Trivial
2425
------------------------------------------------------------------------
2526
-- Functions which preserve equality
2627

28+
-- indexed
2729
record Π {f₁ f₂ t₁ t₂}
2830
(From : Setoid f₁ f₂)
2931
(To : IndexedSetoid (Setoid.Carrier From) t₁ t₂) :
@@ -37,6 +39,7 @@ open Π public
3739

3840
infixr 0 _⟶_
3941

42+
-- not indexed
4043
_⟶_ : {f₁ f₂ t₁ t₂} Setoid f₁ f₂ Setoid t₁ t₂ Set _
4144
From ⟶ To = Π From (Trivial.indexedSetoid To)
4245

@@ -72,6 +75,7 @@ const {B = B} b = record
7275

7376
-- Dependent.
7477

78+
-- indexed
7579
setoid : {f₁ f₂ t₁ t₂}
7680
(From : Setoid f₁ f₂)
7781
IndexedSetoid (Setoid.Carrier From) t₁ t₂
@@ -91,6 +95,7 @@ setoid From To = record
9195

9296
-- Non-dependent.
9397

98+
-- no indexed
9499
infixr 0 _⇨_
95100

96101
_⇨_ : {f₁ f₂ t₁ t₂} Setoid f₁ f₂ Setoid t₁ t₂ Setoid _ _
@@ -99,6 +104,7 @@ From ⇨ To = setoid From (Trivial.indexedSetoid To)
99104
-- A variant of setoid which uses the propositional equality setoid
100105
-- for the domain, and a more convenient definition of _≈_.
101106

107+
-- indexed
102108
≡-setoid : {f t₁ t₂} (From : Set f) IndexedSetoid From t₁ t₂ Setoid _ _
103109
≡-setoid From To = record
104110
{ Carrier = (x : From) Carrier x

src/Relation/Binary/PropositionalEquality.agda

+2-1
Original file line numberDiff line numberDiff line change
@@ -11,7 +11,8 @@ module Relation.Binary.PropositionalEquality where
1111
import Axiom.Extensionality.Propositional as Ext
1212
open import Axiom.UniquenessOfIdentityProofs
1313
open import Function.Base using (id; _∘_)
14-
open import Function.Equality using (Π; _⟶_; ≡-setoid)
14+
open import Function.Equality using (Π; _⟶_)
15+
open import Function.Indexed.Relation.Binary.Equality using (≡-setoid)
1516
open import Level using (Level; _⊔_)
1617
open import Data.Product.Base using (∃)
1718

0 commit comments

Comments
 (0)