Skip to content

Commit 9d1bd5e

Browse files
committed
fix: deprecated definition
1 parent 9070bfd commit 9d1bd5e

File tree

1 file changed

+3
-3
lines changed

1 file changed

+3
-3
lines changed

src/Function/Properties/Surjection.agda

Lines changed: 3 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -12,8 +12,8 @@ open import Function.Base using (_∘_; _$_)
1212
open import Function.Definitions using (Surjective; Injective; Congruent)
1313
open import Function.Bundles
1414
using (Func; Surjection; _↠_; _⟶_; _↪_; mk↪; _⇔_; mk⇔)
15+
open import Function.Consequences using (module Section)
1516
import Function.Construct.Identity as Identity
16-
import Function.Construct.Symmetry as Symmetry
1717
import Function.Construct.Composition as Compose
1818
open import Level using (Level)
1919
open import Data.Product.Base using (_,_; proj₁; proj₂)
@@ -46,7 +46,7 @@ mkSurjection f surjective = record
4646
↠⇒⟶ = Surjection.function
4747

4848
↠⇒↪ : A ↠ B B ↪ A
49-
↠⇒↪ s = mk↪ {from = to} λ { ≡.refl section-strictInverseˡ _ }
49+
↠⇒↪ s = mk↪ {from = to} λ { ≡.refl strictlyInverseˡ _ }
5050
where open Surjection s
5151

5252
↠⇒⇔ : A ↠ B A ⇔ B
@@ -80,7 +80,7 @@ module _ (surjection : Surjection S T) where
8080
injective⇒to⁻-cong : Injective Eq₁._≈_ Eq₂._≈_ to
8181
Congruent Eq₂._≈_ Eq₁._≈_ section
8282
injective⇒to⁻-cong injective =
83-
Symmetry.section-cong (injective , surjective) Eq₁.refl Eq₂.sym Eq₂.trans
83+
Section.cong Eq₂._≈_ surjective injective Eq₁.refl Eq₂.sym Eq₂.trans
8484
{-# WARNING_ON_USAGE injective⇒to⁻-cong
8585
"Warning: injective⇒to⁻-cong was deprecated in v2.3.
8686
Please use Symmetry.section-cong instead. "

0 commit comments

Comments
 (0)