We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 355ac25 commit cc69ea0Copy full SHA for cc69ea0
src/Data/List/Relation/Unary/All.agda
@@ -115,7 +115,7 @@ zip = zipWith id
115
unzip : All (P ∩ Q) ⊆ All P ∩ All Q
116
unzip = unzipWith id
117
118
-module _(S : Setoid a ℓ) {P : Pred (Setoid.Carrier S) p} where
+module _ (S : Setoid a ℓ) {P : Pred (Setoid.Carrier S) p} where
119
open Setoid S renaming (refl to ≈-refl)
120
open SetoidMembership S
121
0 commit comments