Skip to content

Commit

Permalink
Update src/Init/Core.lean
Browse files Browse the repository at this point in the history
Co-authored-by: Kyle Miller <kmill31415@gmail.com>
  • Loading branch information
joehendrix and kmill authored Jan 22, 2024
1 parent b27bc26 commit ad84c63
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion src/Init/Core.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1762,7 +1762,7 @@ proof.
This class is intended for simplifying defining instances of
`LawfulIdentity` and functions needed commutative operations with
identity should just add a `LawfulIdentity constraint.
identity should just add a `LawfulIdentity` constraint.
-/
class LawfulCommIdentity (op : α → α → α) (o : outParam α) [hc : Commutative op] extends LawfulIdentity op o : Prop where
left_id a := Eq.trans (hc.comm o a) (right_id a)
Expand Down

0 comments on commit ad84c63

Please sign in to comment.