Skip to content

Commit

Permalink
chore(linear_algebra/dual): prove a lemma with rfl (#18444)
Browse files Browse the repository at this point in the history
I was surprised that `dsimp` didn't clean this up for me.
The proof that used to be here was certainly not interesting.
  • Loading branch information
eric-wieser committed Feb 16, 2023
1 parent 10d8872 commit 5455cb0
Showing 1 changed file with 1 addition and 5 deletions.
6 changes: 1 addition & 5 deletions src/linear_algebra/dual.lean
Expand Up @@ -118,11 +118,7 @@ instance : has_coe_to_fun (dual R M) (λ _, M → R) := ⟨linear_map.to_fun⟩
`module.eval_equiv`. -/
def eval : M →ₗ[R] (dual R (dual R M)) := linear_map.flip linear_map.id

@[simp] lemma eval_apply (v : M) (a : dual R M) : eval R M v a = a v :=
begin
dunfold eval,
rw [linear_map.flip_apply, linear_map.id_apply]
end
@[simp] lemma eval_apply (v : M) (a : dual R M) : eval R M v a = a v := rfl

variables {R M} {M' : Type*} [add_comm_monoid M'] [module R M']

Expand Down

0 comments on commit 5455cb0

Please sign in to comment.