Skip to content

Commit

Permalink
Revert "feat: add support for not-in in exists (#425)" (#427)
Browse files Browse the repository at this point in the history
This `binder_predicate` is already defined in another file, and so this causes ambiguity in the grammar.
  • Loading branch information
tobiasgrosser authored Dec 8, 2023
1 parent 63c387d commit b197bd2
Showing 1 changed file with 0 additions and 2 deletions.
2 changes: 0 additions & 2 deletions Std/Util/ExtendedBinder.lean
Original file line number Diff line number Diff line change
Expand Up @@ -138,5 +138,3 @@ binder_predicate x " < " y:term => `($x < $y)
binder_predicate x " ≤ " y:term => `($x ≤ $y)
/-- Declare `∃ x ≠ y, ...` as syntax for `∃ x, x ≠ y ∧ ...` -/
binder_predicate x " ≠ " y:term => `($x ≠ $y)
/-- Declare `∃ x ∉ y, ...` as syntax for `∃ x, x ∉ y ∧ ...` -/
binder_predicate x " ∉ " y:term => `($x ∉ $y)

0 comments on commit b197bd2

Please sign in to comment.