Skip to content

Commit

Permalink
chore(*): fix last line length and notation style linter errors (#10642)
Browse files Browse the repository at this point in the history
These are the last non-module doc style linter errors (from https://github.com/leanprover-community/mathlib/blob/master/scripts/style-exceptions.txt).



Co-authored-by: Rob Lewis <rob.y.lewis@gmail.com>
  • Loading branch information
robertylewis and robertylewis committed Dec 7, 2021
1 parent cd857f7 commit 9031989
Show file tree
Hide file tree
Showing 6 changed files with 11 additions and 6 deletions.
3 changes: 2 additions & 1 deletion src/data/pfunctor/multivariate/M.lean
Expand Up @@ -40,7 +40,8 @@ that `A` is a possibly infinite tree.
## Reference
* [Jeremy Avigad, Mario M. Carneiro and Simon Hudon, *Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
* Jeremy Avigad, Mario M. Carneiro and Simon Hudon.
[*Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
-/

universe u
Expand Down
3 changes: 2 additions & 1 deletion src/data/pfunctor/multivariate/W.lean
Expand Up @@ -39,7 +39,8 @@ its valid paths to values of `α`
## Reference
* [Jeremy Avigad, Mario M. Carneiro and Simon Hudon, *Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
* Jeremy Avigad, Mario M. Carneiro and Simon Hudon.
[*Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
-/

universes u v
Expand Down
3 changes: 2 additions & 1 deletion src/data/qpf/multivariate/constructions/cofix.lean
Expand Up @@ -35,7 +35,8 @@ We define the relation `Mcongr` and take its quotient as the definition of `cofi
## Reference
* [Jeremy Avigad, Mario M. Carneiro and Simon Hudon, *Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
* Jeremy Avigad, Mario M. Carneiro and Simon Hudon.
[*Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
-/

universe u
Expand Down
3 changes: 2 additions & 1 deletion src/data/qpf/multivariate/constructions/fix.lean
Expand Up @@ -44,7 +44,8 @@ See [avigad-carneiro-hudon2019] for more details.
## Reference
* [Jeremy Avigad, Mario M. Carneiro and Simon Hudon, *Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
* Jeremy Avigad, Mario M. Carneiro and Simon Hudon.
[*Data Types as Quotients of Polynomial Functors*][avigad-carneiro-hudon2019]
-/

universes u v
Expand Down
2 changes: 0 additions & 2 deletions src/tactic/induction.lean
Expand Up @@ -1325,8 +1325,6 @@ meta def generalisation_mode_parser : lean.parser generalization_mode :=
<|>
pure (generalization_mode.generalize_all_except [])

precedence `fixing`:0

/--
A variant of `tactic.interactive.induction`, with the following differences:
Expand Down
3 changes: 3 additions & 0 deletions src/tactic/reserved_notation.lean
Expand Up @@ -47,6 +47,9 @@ reserve notation `to`
-- used in `tactic/rcases.lean`
precedence `?`:max

-- used in `tactic/induction.lean`
precedence `fixing`:0

-- used in `order/lattice.lean`
reserve infixl ` ⊓ `:70
reserve infixl ` ⊔ `:65
Expand Down

0 comments on commit 9031989

Please sign in to comment.