Skip to content

Commit

Permalink
chore: unused variable warnings (#52)
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em authored Oct 11, 2024
1 parent 505974b commit 313a82f
Show file tree
Hide file tree
Showing 2 changed files with 2 additions and 2 deletions.
2 changes: 1 addition & 1 deletion Tests.lean
Original file line number Diff line number Diff line change
Expand Up @@ -45,7 +45,7 @@ def heya : IO Unit := do
if x == 3 /-
!! begin foo
-/ || true /- !! end foo -/ then pure ()
let x := [1, 2/- !! begin foo-/, 3/- !! end foo-/]
let _ := [1, 2/- !! begin foo-/, 3/- !! end foo-/]
pure ()

def expectedLog :=
Expand Down
2 changes: 1 addition & 1 deletion src/highlighting/SubVerso/Highlighting/Code.lean
Original file line number Diff line number Diff line change
Expand Up @@ -93,7 +93,7 @@ instance [h1 : Nonempty α] [h2 : Nonempty β] : Nonempty (α × β) :=
⟨(x, y)⟩


example [Inhabited α] [Monad m] [MonadState (State α) m] [BEq α] [Hashable α] (x : α) : Inhabited (m (Nat × α × Nat)) := inferInstance
example [Inhabited α] [Monad m] [MonadState (State α) m] [BEq α] [Hashable α] (_ : α) : Inhabited (m (Nat × α × Nat)) := inferInstance

-- Lifted from find's where block to make sure the Inhabited instance is found
partial def find.loop [Inhabited α] [Monad m] [MonadState (State α) m] (i : Nat) : m (Nat × α × Nat) := do
Expand Down

0 comments on commit 313a82f

Please sign in to comment.