Skip to content

Commit

Permalink
add @[inherit_doc] to equiv notation (#7998)
Browse files Browse the repository at this point in the history
This makes hovering over `≃` display the docstring for `Equiv` (if I've understood things correctly).
  • Loading branch information
kbuzzard committed Oct 28, 2023
1 parent d70b029 commit 2aead33
Showing 1 changed file with 1 addition and 0 deletions.
1 change: 1 addition & 0 deletions Mathlib/Logic/Equiv/Defs.lean
Expand Up @@ -70,6 +70,7 @@ structure Equiv (α : Sort*) (β : Sort _) where
protected right_inv : RightInverse invFun toFun
#align equiv Equiv

@[inherit_doc]
infixl:25 " ≃ " => Equiv

/-- Turn an element of a type `F` satisfying `EquivLike F α β` into an actual
Expand Down

0 comments on commit 2aead33

Please sign in to comment.