Skip to content

Commit

Permalink
[v2.1-rc1] fixes #2400: use explicit quantification instead (#2429)
Browse files Browse the repository at this point in the history
* fixes #2400: use explicit quantification

* fix knock-ons
  • Loading branch information
jamesmckinna authored Jul 5, 2024
1 parent 606bea8 commit 848d8e8
Show file tree
Hide file tree
Showing 2 changed files with 8 additions and 8 deletions.
8 changes: 4 additions & 4 deletions src/Function/Endo/Setoid.agda
Original file line number Diff line number Diff line change
Expand Up @@ -58,7 +58,7 @@ private
∘-isMagma : IsMagma _≈_ _∘_
∘-isMagma = record
{ isEquivalence = isEquivalence
; ∙-cong = λ {_} {_} {_} {v} x≈y u≈v S.trans u≈v (cong v x≈y)
; ∙-cong = λ {_} {_} {_} {k} f≈g h≈k x S.trans (h≈k _) (cong k (f≈g x))
}

∘-magma : Magma (c ⊔ e) (c ⊔ e)
Expand All @@ -67,7 +67,7 @@ private
∘-isSemigroup : IsSemigroup _≈_ _∘_
∘-isSemigroup = record
{ isMagma = ∘-isMagma
; assoc = λ _ _ _ S.refl
; assoc = λ _ _ _ _ S.refl
}

∘-semigroup : Semigroup (c ⊔ e) (c ⊔ e)
Expand All @@ -76,7 +76,7 @@ private
∘-id-isMonoid : IsMonoid _≈_ _∘_ id
∘-id-isMonoid = record
{ isSemigroup = ∘-isSemigroup
; identity = (λ _ S.refl) , (λ _ S.refl)
; identity = (λ _ _ S.refl) , (λ _ _ S.refl)
}

∘-id-monoid : Monoid (c ⊔ e) (c ⊔ e)
Expand Down Expand Up @@ -112,6 +112,6 @@ module _ (f : Endo) where
^-isMonoidHomomorphism : IsMonoidHomomorphism +-0-rawMonoid ∘-id-rawMonoid (f ^_)
^-isMonoidHomomorphism = record
{ isMagmaHomomorphism = ^-isMagmaHomomorphism
; ε-homo = S.refl
; ε-homo = λ _ S.refl
}

8 changes: 4 additions & 4 deletions src/Function/Relation/Binary/Setoid/Equality.agda
Original file line number Diff line number Diff line change
Expand Up @@ -24,16 +24,16 @@ private

infix 4 _≈_
_≈_ : (f g : Func From To) Set (a₁ ⊔ b₂)
f ≈ g = {x : From.Carrier} f ⟨$⟩ x To.≈ g ⟨$⟩ x
f ≈ g = x f ⟨$⟩ x To.≈ g ⟨$⟩ x

refl : Reflexive _≈_
refl = To.refl
refl _ = To.refl

sym : Symmetric _≈_
sym = λ f≈g To.sym f≈g
sym f≈g x = To.sym (f≈g x)

trans : Transitive _≈_
trans = λ f≈g g≈h To.trans f≈g g≈h
trans f≈g g≈h x = To.trans (f≈g x) (g≈h x)

isEquivalence : IsEquivalence _≈_
isEquivalence = record -- need to η-expand else Agda gets confused
Expand Down

0 comments on commit 848d8e8

Please sign in to comment.