Skip to content

Commit

Permalink
feat(Data/Opposite): Show that op, unop are surjective (#11240)
Browse files Browse the repository at this point in the history
  • Loading branch information
uniwuni authored and utensil committed Mar 26, 2024
1 parent 6d8ec38 commit d4c2327
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions Mathlib/Data/Opposite.lean
Original file line number Diff line number Diff line change
Expand Up @@ -89,6 +89,10 @@ def equivToOpposite : α ≃ αᵒᵖ where
right_inv := op_unop
#align opposite.equiv_to_opposite Opposite.equivToOpposite

theorem op_surjective : Function.Surjective (op : α → αᵒᵖ) := equivToOpposite.surjective

theorem unop_surjective : Function.Surjective (unop : αᵒᵖ → α) := equivToOpposite.symm.surjective

@[simp]
theorem equivToOpposite_coe : (equivToOpposite : α → αᵒᵖ) = op :=
rfl
Expand Down

0 comments on commit d4c2327

Please sign in to comment.