Skip to content

Commit

Permalink
chore(algebra/group/basic): Mark inv_involutive simp (#4744)
Browse files Browse the repository at this point in the history
This means expressions like `has_inv.inv ∘ has_inv.inv` can be simplified
  • Loading branch information
eric-wieser committed Oct 23, 2020
1 parent bb52355 commit 458c833
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/algebra/group/basic.lean
Expand Up @@ -95,7 +95,7 @@ theorem left_inverse_inv (G) [group G] :
function.left_inverse (λ a : G, a⁻¹) (λ a, a⁻¹) :=
inv_inv

@[to_additive]
@[simp, to_additive]
lemma inv_involutive : function.involutive (has_inv.inv : G → G) := inv_inv

@[to_additive]
Expand Down

0 comments on commit 458c833

Please sign in to comment.