diff --git a/src/Function/Endo/Setoid.agda b/src/Function/Endo/Setoid.agda index 99716b35db..583ba2f4c6 100644 --- a/src/Function/Endo/Setoid.agda +++ b/src/Function/Endo/Setoid.agda @@ -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) @@ -67,7 +67,7 @@ private ∘-isSemigroup : IsSemigroup _≈_ _∘_ ∘-isSemigroup = record { isMagma = ∘-isMagma - ; assoc = λ _ _ _ → S.refl + ; assoc = λ _ _ _ _ → S.refl } ∘-semigroup : Semigroup (c ⊔ e) (c ⊔ e) @@ -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) @@ -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 } diff --git a/src/Function/Relation/Binary/Setoid/Equality.agda b/src/Function/Relation/Binary/Setoid/Equality.agda index 9d0e9823da..6c530b0e9b 100644 --- a/src/Function/Relation/Binary/Setoid/Equality.agda +++ b/src/Function/Relation/Binary/Setoid/Equality.agda @@ -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