Skip to content

Commit

Permalink
chore(RingTheory/WittVector/Basic): remove porting notes (#13927)
Browse files Browse the repository at this point in the history
Remove a couple uncategorised, superfluous porting notes.
  • Loading branch information
joneugster committed Jun 18, 2024
1 parent 6f05744 commit b84002d
Showing 1 changed file with 2 additions and 9 deletions.
11 changes: 2 additions & 9 deletions Mathlib/RingTheory/WittVector/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -158,7 +158,6 @@ private def ghostFun : π•Ž R β†’ β„• β†’ R := fun x n => aeval x.coeff (W_ β„€
section Tactic
open Lean Elab Tactic

-- porting note: removed mathport output related to meta code.
/-- An auxiliary tactic for proving that `ghostFun` respects the ring operations. -/
elab "ghost_fun_tac" Ο†:term "," fn:term : tactic => do
evalTactic (← `(tactic| (
Expand Down Expand Up @@ -219,14 +218,10 @@ private theorem ghostFun_intCast (i : β„€) : ghostFun (i : π•Ž R) = i :=
alias ghostFun_int_cast := ghostFun_intCast

private lemma ghostFun_nsmul (m : β„•) (x : WittVector p R) : ghostFun (m β€’ x) = m β€’ ghostFun x := by
-- porting note: I had to add the explicit type ascription.
-- This could very well be due to my poor tactic writing!
ghost_fun_tac m β€’ (X 0 : MvPolynomial _ β„€), ![x.coeff]
ghost_fun_tac m β€’ (X 0), ![x.coeff]

private lemma ghostFun_zsmul (m : β„€) (x : WittVector p R) : ghostFun (m β€’ x) = m β€’ ghostFun x := by
-- porting note: I had to add the explicit type ascription.
-- This could very well be due to my poor tactic writing!
ghost_fun_tac m β€’ (X 0 : MvPolynomial _ β„€), ![x.coeff]
ghost_fun_tac m β€’ (X 0), ![x.coeff]

private theorem ghostFun_pow (m : β„•) : ghostFun (x ^ m) = ghostFun x ^ m := by
ghost_fun_tac X 0 ^ m, ![x.coeff]
Expand Down Expand Up @@ -256,8 +251,6 @@ private def ghostEquiv' [Invertible (p : R)] : π•Ž R ≃ (β„• β†’ R) where

@[local instance]
private def comm_ring_aux₁ : CommRing (π•Ž (MvPolynomial R β„š)) :=
-- Porting note: no longer needed?
-- letI : CommRing (MvPolynomial R β„š) := MvPolynomial.commRing
(ghostEquiv' p (MvPolynomial R β„š)).injective.commRing ghostFun ghostFun_zero ghostFun_one
ghostFun_add ghostFun_mul ghostFun_neg ghostFun_sub ghostFun_nsmul ghostFun_zsmul
ghostFun_pow ghostFun_natCast ghostFun_intCast
Expand Down

0 comments on commit b84002d

Please sign in to comment.