@@ -12,8 +12,8 @@ open import Function.Base using (_∘_; _$_)
12
12
open import Function.Definitions using (Surjective; Injective; Congruent)
13
13
open import Function.Bundles
14
14
using (Func; Surjection; _↠_; _⟶_; _↪_; mk↪; _⇔_; mk⇔)
15
+ open import Function.Consequences using (module Section )
15
16
import Function.Construct.Identity as Identity
16
- import Function.Construct.Symmetry as Symmetry
17
17
import Function.Construct.Composition as Compose
18
18
open import Level using (Level)
19
19
open import Data.Product.Base using (_,_; proj₁; proj₂)
@@ -46,7 +46,7 @@ mkSurjection f surjective = record
46
46
↠⇒⟶ = Surjection.function
47
47
48
48
↠⇒↪ : A ↠ B → B ↪ A
49
- ↠⇒↪ s = mk↪ {from = to} λ { ≡.refl → section-strictInverseˡ _ }
49
+ ↠⇒↪ s = mk↪ {from = to} λ { ≡.refl → strictlyInverseˡ _ }
50
50
where open Surjection s
51
51
52
52
↠⇒⇔ : A ↠ B → A ⇔ B
@@ -80,7 +80,7 @@ module _ (surjection : Surjection S T) where
80
80
injective⇒to⁻-cong : Injective Eq₁._≈_ Eq₂._≈_ to →
81
81
Congruent Eq₂._≈_ Eq₁._≈_ section
82
82
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
84
84
{-# WARNING_ON_USAGE injective⇒to⁻-cong
85
85
"Warning: injective⇒to⁻-cong was deprecated in v2.3.
86
86
Please use Symmetry.section-cong instead. "
0 commit comments