Skip to content

Commit

Permalink
doc(Tactic/Ring/Basic): fix documentation for ExProd.mkRat (#22180)
Browse files Browse the repository at this point in the history
Co-authored-by: Daniel Weber <[email protected]>
  • Loading branch information
Command-Master and Command-Master committed Feb 25, 2025
1 parent 6d33eaf commit c265423
Showing 1 changed file with 2 additions and 1 deletion.
3 changes: 2 additions & 1 deletion Mathlib/Tactic/Ring/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -265,7 +265,8 @@ def ExProd.mkNegNat (_ : Q(Ring $α)) (n : ℕ) : (e : Q($α)) × ExProd sα e :
⟨q((Int.negOfNat $lit).rawCast : $α), .const (-n) none⟩

/--
Constructs the expression corresponding to `.const (-n)`.
Constructs the expression corresponding to `.const q h` for `q = n / d`
and `h` a proof that `(d : α) ≠ 0`.
(The `.const` constructor does not check that the expression is correct.)
-/
def ExProd.mkRat (_ : Q(DivisionRing $α)) (q : ℚ) (n : Q(ℤ)) (d : Q(ℕ)) (h : Expr) :
Expand Down

0 comments on commit c265423

Please sign in to comment.