Skip to content

Commit

Permalink
.
Browse files Browse the repository at this point in the history
  • Loading branch information
artie2000 authored Jan 22, 2025
1 parent 702e49c commit 4128908
Showing 1 changed file with 1 addition and 1 deletion.
2 changes: 1 addition & 1 deletion Mathlib/Algebra/Ring/Subring/Defs.lean
Original file line number Diff line number Diff line change
Expand Up @@ -85,7 +85,7 @@ instance (priority := 100) SubringClass.nonUnitalSubringClass (S : Type*) (R : T

variable [SetLike S R] [hSR : SubringClass S R] (s : S)

@[simp]
@[simp, aesop safe apply (rule_sets := [SetLike])]
theorem intCast_mem (n : ℤ) : (n : R) ∈ s := by simp only [← zsmul_one, zsmul_mem, one_mem]

@[deprecated _root_.intCast_mem (since := "2024-04-05")] alias coe_int_mem := intCast_mem
Expand Down

0 comments on commit 4128908

Please sign in to comment.