leanprover-community / mathlib

  • Home
  • Zulip archive
  • API documentation
  • Lean web editor
  • Links

Zulip Chat Archive

Stream: new members

Topic: Turn implicitly declared variables explicit in definition


Vivek Rajesh Joshi (Aug 18 2024 at 16:11):

import Mathlib.Data.Matrix.Notation

variable {F : Type} [Field F] [DecidableEq F]

-- [0,0,..(z times)..,0,first_nz,[tail]]
structure row (F : Type) [Field F] [DecidableEq F] where
  z : Nat
  first_nz : F
  tail : List F

Is there a shorter, cleaner way to make F an implicit parameter in row?


Last updated: May 02 2025 at 03:31 UTC

Theme Simple by wildflame © 2016 Powered by jekyll