Zulip Chat Archive

Stream: new members

Topic: Remove decide ... = true from Bool hypothesis


Vivek Rajesh Joshi (May 17 2024 at 13:56):

import Mathlib.Data.Matrix.Notation
variable (M : Matrix (Fin m) (Fin n) Rat) (hm : m>0) (hn : n>0)

abbrev colListofMat := List.map List.ofFn (List.ofFn M.transpose)

def list_allZero (l : List Rat) : Bool := l.all (fun x => (x==0))

def findNonzCol :  := (colListofMat M).findIdx (fun col => ¬ list_allZero col)

lemma findNonzCol_get_HasNonz (h : findNonzCol M < (colListofMat M).length) :
   x  (colListofMat M).get findNonzCol M,h⟩, x0 := by
  have := List.findIdx_get (w:=h)

What can I do to to get rid of the decide ... = true in this?

Yaël Dillies (May 17 2024 at 13:59):

simp at this

Vivek Rajesh Joshi (May 17 2024 at 14:01):

It also simplifies some other definitions that I don't want simplified. How do I specifically simplify the decide part?

Vivek Rajesh Joshi (May 17 2024 at 14:01):

Nvm, simp? at this tells me what I want. Thanks anyways!


Last updated: May 02 2025 at 03:31 UTC