File tree Expand file tree Collapse file tree 2 files changed +7
-9
lines changed Expand file tree Collapse file tree 2 files changed +7
-9
lines changed Original file line number Diff line number Diff line change @@ -199,14 +199,12 @@ public export
199199TyName' : KeyVal
200200TyName' = " name" :-: FCBind Name
201201
202- namespace TypeName
203- ||| Extract the "tyname" value from the metadata record
204- export
205- (. tyName) : {n : Nat } ->
206- (inRange : NameInRange "name" fields === Just (n, FCBind Name )) =>
207- WithData fields a -> FCBind Name
208- (. tyName) = WithData . get " name" @{inRange}
209-
202+ ||| Extract the "tyname" value from the metadata record
203+ export
204+ (. tyName) : {n : Nat } ->
205+ (inRange : NameInRange "name" fields === Just (n, FCBind Name )) =>
206+ WithData fields a -> FCBind Name
207+ (. tyName) = WithData . get " name" @{inRange}
210208
211209||| Attach documentation, binding and location information to a type
212210public export
Original file line number Diff line number Diff line change @@ -190,7 +190,7 @@ getMethToplevel {vars} env vis iname cname constraints allmeths bindNames params
190190 let tydecl = IClaim (MkFCVal vfc $ MkIClaimData sig. count vis (if sig. isData then [Inline , Invertible ]
191191 else [Inline ])
192192 (Mk [vfc, NotBinding : + cn] ty_imp))
193- let conapp = apply (IVar vfc cname) (map (IBindVar EmptyFC ) allmeths )
193+ let conapp = apply (IVar vfc cname) (map (IBindVar EmptyFC ) bindNames )
194194 let argns = getExplicitArgs 0 sig. type
195195 -- eta expand the RHS so that we put implicits in the right place
196196 let fnclause = PatClause vfc
You can’t perform that action at this time.
0 commit comments