Skip to content

Commit

Permalink
fixes #2467 (#2468)
Browse files Browse the repository at this point in the history
  • Loading branch information
jamesmckinna authored Aug 30, 2024
1 parent 355ac25 commit cc69ea0
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Data/List/Relation/Unary/All.agda
Original file line number Diff line number Diff line change
Expand Up @@ -115,7 +115,7 @@ zip = zipWith id
unzip : All (P ∩ Q) ⊆ All P ∩ All Q
unzip = unzipWith id

module _(S : Setoid a ℓ) {P : Pred (Setoid.Carrier S) p} where
module _ (S : Setoid a ℓ) {P : Pred (Setoid.Carrier S) p} where
open Setoid S renaming (refl to ≈-refl)
open SetoidMembership S

Expand Down

0 comments on commit cc69ea0

Please sign in to comment.