Skip to content

Commit f664387

Browse files
committed
Remove some explicitly bound variables in type signatures
1 parent 2631807 commit f664387

File tree

2 files changed

+2
-4
lines changed

2 files changed

+2
-4
lines changed

src/Data/Product/Function/Dependent/Propositional.agda

Lines changed: 1 addition & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -317,7 +317,5 @@ cong {B = B} {k = leftInverse} I↔J A↩B = ↩⇒↪ (Σ-↩ (↔⇒↩
317317
cong {k = surjection} I↔J A↠B = Σ-↠ (↔⇒↠ I↔J) A↠B
318318
cong {k = bijection} I↔J A↔B = Σ-↔ I↔J A↔B
319319

320-
cong′ : {k} {A : Set a} {B₁ : A Set b} {B₂ : A Set c}
321-
( {x} B₁ x ∼[ k ] B₂ x)
322-
Σ A B₁ ∼[ k ] Σ A B₂
320+
cong′ : {k} ( {x} A x ∼[ k ] B x) Σ I A ∼[ k ] Σ I B
323321
cong′ = cong (refl _)

src/Function/Related/TypeIsomorphisms.agda

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -357,6 +357,6 @@ True↔ (false because ofⁿ ¬p) _ =
357357
-- Relating a predicate to an existentially quantified one with the
358358
-- restriction that the quantified variable is equal to the given one
359359

360-
∃-≡ : {A : Set a} (P : A Set b) {x} P x ↔ (∃[ y ] y ≡ x × P y)
360+
∃-≡ : (P : A Set b) {x} P x ↔ (∃[ y ] y ≡ x × P y)
361361
∃-≡ P {x} = mk↔ₛ′ (λ Px x , refl , Px) (λ where (_ , (refl , Py)) Py)
362362
(λ where (_ , refl , _) refl) (λ where _ refl)

0 commit comments

Comments
 (0)