Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit ae1b530

Browse files
committed
chore(algebra/algebra/basic): add simp lemma about algebra_map ℚ (#5970)
Since there is a subsingleton instance over ring_homs, we may as well let the simplifier replace `algebra_map` with `id`.
1 parent f596077 commit ae1b530

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/algebra/algebra/basic.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1013,6 +1013,9 @@ namespace rat
10131013
instance algebra_rat {α} [division_ring α] [char_zero α] : algebra ℚ α :=
10141014
(rat.cast_hom α).to_algebra' $ λ r x, r.cast_commute x
10151015

1016+
@[simp] theorem algebra_map_rat_rat : algebra_map ℚ ℚ = ring_hom.id ℚ :=
1017+
subsingleton.elim _ _
1018+
10161019
end rat
10171020

10181021
namespace algebra

0 commit comments

Comments
 (0)