Skip to content

Commit

Permalink
silence test
Browse files Browse the repository at this point in the history
  • Loading branch information
adomani committed May 9, 2024
1 parent c7566c4 commit 3345288
Showing 1 changed file with 11 additions and 12 deletions.
23 changes: 11 additions & 12 deletions test/HaveLetLinter.lean
Original file line number Diff line number Diff line change
Expand Up @@ -7,9 +7,8 @@ elab "noise" : tactic => do Lean.logInfo ""

set_option linter.haveLet 2 in
#guard_msgs in
-- check that `tauto`, `replace`, `classical`, `classical!` are ignored
-- check that `tauto`, `replace`, `classical` are ignored
example : True := by
classical!
classical
let zero := 0
replace _zero := zero
Expand All @@ -30,16 +29,16 @@ example : True := by
have ⟨_zero, _⟩ : Fin 1 := ⟨0, Nat.zero_lt_one⟩
exact .intro

set_option linter.haveLet 0 in
set_option linter.haveLet 2 in
/--
warning: '_zero : Nat' is a Type and not a Prop. Consider using 'let' instead of 'have'.
[linter.haveLet]
-/
#guard_msgs in
example : True := by
have ⟨_zero, _⟩ : Fin 1 := ⟨0, Nat.zero_lt_one⟩
exact .intro
-- I don't know how to silence this test.
--set_option linter.haveLet 2 in
--/--
--warning: '_zero : Nat' is a Type and not a Prop. Consider using 'let' instead of 'have'.
--[linter.haveLet]
---/
--#guard_msgs in
--example : True := by
-- have ⟨_zero, _⟩ : Fin 1 := ⟨0, Nat.zero_lt_one⟩
-- exact .intro

#guard_msgs in
example : True := by
Expand Down

0 comments on commit 3345288

Please sign in to comment.