Skip to content

Commit

Permalink
Try to remove some nolints
Browse files Browse the repository at this point in the history
  • Loading branch information
nomeata committed Aug 21, 2024
1 parent 0cbb129 commit 4b976ec
Show file tree
Hide file tree
Showing 2 changed files with 0 additions and 3 deletions.
2 changes: 0 additions & 2 deletions Mathlib/Computability/Primrec.lean
Original file line number Diff line number Diff line change
Expand Up @@ -58,8 +58,6 @@ namespace Nat
@[simp, reducible]
def unpaired {α} (f : ℕ → ℕ → α) (n : ℕ) : α :=
f n.unpair.1 n.unpair.2
attribute [nolint simpVarHead] unpaired.eq_1


/-- The primitive recursive functions `ℕ → ℕ`. -/
protected inductive Primrec : (ℕ → ℕ) → Prop
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Logic/Function/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -25,7 +25,6 @@ variable {α β γ : Sort*} {f : α → β}
/-- Evaluate a function at an argument. Useful if you want to talk about the partially applied
`Function.eval x : (∀ x, β x) → β x`. -/
@[reducible, simp] def eval {β : α → Sort*} (x : α) (f : ∀ x, β x) : β x := f x
attribute [nolint simpVarHead] eval.eq_1

theorem eval_apply {β : α → Sort*} (x : α) (f : ∀ x, β x) : eval x f = f x :=
rfl
Expand Down

0 comments on commit 4b976ec

Please sign in to comment.