Skip to content

Commit

Permalink
Fix setOption linter in tests: mostly disable it; in one instance, on…
Browse files Browse the repository at this point in the history
…e option could be simply removed.
  • Loading branch information
grunweg committed May 22, 2024
1 parent b9903b0 commit b683b75
Show file tree
Hide file tree
Showing 7 changed files with 6 additions and 2 deletions.
1 change: 1 addition & 0 deletions test/Explode.lean
Original file line number Diff line number Diff line change
Expand Up @@ -24,6 +24,7 @@ info: true_iff : ∀ (p : Prop), (True ↔ p) = p
-/
#guard_msgs in #explode true_iff

set_option linter.setOption false
-- On command line, tests format functions with => rather than ↦ without this.
set_option pp.unicode.fun true

Expand Down
2 changes: 0 additions & 2 deletions test/LibrarySearch/IsCompact.lean
Original file line number Diff line number Diff line change
@@ -1,8 +1,6 @@
import Mathlib.Topology.Instances.Real
import Mathlib.Topology.Algebra.Order.Compact

set_option pp.unicode.fun true

-- TODO: uses sorry, but is hidden behind the `apply?`
/-- warning: declaration uses 'sorry' -/
#guard_msgs(warning, drop info) in
Expand Down
1 change: 1 addition & 0 deletions test/LibrarySearch/basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,6 +6,7 @@ import Mathlib.Data.Real.Basic

set_option autoImplicit true

set_option linter.setOption false
-- Enable this option for tracing:
-- set_option trace.Tactic.librarySearch true
-- And this option to trace all candidate lemmas before application.
Expand Down
1 change: 1 addition & 0 deletions test/Recall.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,6 +3,7 @@ import Mathlib.Analysis.Calculus.Deriv.Basic
import Mathlib.Analysis.SpecialFunctions.Trigonometric.Basic
import Mathlib.Data.Complex.Exponential

set_option linter.setOption false
-- Remark: When the test is run by make/CI, this option is not set, so we set it here.
set_option pp.unicode.fun true
set_option autoImplicit true
Expand Down
1 change: 1 addition & 0 deletions test/delabLinearIndependent.lean
Original file line number Diff line number Diff line change
@@ -1,5 +1,6 @@
import Mathlib.LinearAlgebra.LinearIndependent

set_option linter.setOption false
set_option pp.unicode.fun true

variable {K V : Type*} [DivisionRing K] [AddCommGroup V] [Module K V] {s : Set V} {x : V}
Expand Down
1 change: 1 addition & 0 deletions test/linarith.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,7 @@ import Mathlib.Data.Rat.Order
private axiom test_sorry : ∀ {α}, α
set_option linter.unusedVariables false
set_option autoImplicit true
set_option linter.setOption false
set_option pp.mvars false

example [LinearOrderedCommRing α] {a b : α} (h : a < b) (w : b < a) : False := by
Expand Down
1 change: 1 addition & 0 deletions test/vec_notation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,6 +8,7 @@ open Lean
open Lean.Meta
open Qq

set_option linter.setOption false in
set_option pp.unicode.fun false

/-! These tests are testing `PiFin.toExpr` and fail with
Expand Down

0 comments on commit b683b75

Please sign in to comment.