Skip to content

Commit

Permalink
chore: remove binder_predicate (#817)
Browse files Browse the repository at this point in the history
It has been upstreamed to Lean4.
  • Loading branch information
FR-vdash-bot authored Jun 3, 2024
1 parent dfe8208 commit ee87917
Showing 1 changed file with 0 additions and 19 deletions.
19 changes: 0 additions & 19 deletions Batteries/Util/ExtendedBinder.lean
Original file line number Diff line number Diff line change
Expand Up @@ -52,22 +52,3 @@ macro_rules -- TODO: merging the two macro_rules breaks expansion
| `(∀ᵉ _ : $ty:term, $b) => `(∀ _ : $ty:term, $b)
| `(∀ᵉ $x:ident : $ty:term, $b) => `(∀ $x:ident : $ty:term, $b)
| `(∀ᵉ $x:binderIdent $p:binderPred, $b) => `(∀ $x:binderIdent $p:binderPred, $b)

open Parser.Command in
/--
Declares a binder predicate. For example:
```
binder_predicate x " > " y:term => `($x > $y)
```
-/
syntax (name := binderPredicate) (docComment)? (Parser.Term.attributes)? (attrKind)?
"binder_predicate" optNamedName optNamedPrio ppSpace ident (ppSpace macroArg)* " => "
term : command

open Linter.MissingDocs Parser Term in
/-- Missing docs handler for `binder_predicate` -/
@[missing_docs_handler binderPredicate]
def checkBinderPredicate : SimpleHandler := fun stx => do
if stx[0].isNone && stx[2][0][0].getKind != ``«local» then
if stx[4].isNone then lint stx[3] "binder predicate"
else lintNamed stx[4][0][3] "binder predicate"

0 comments on commit ee87917

Please sign in to comment.