function relating the offbrand notions of chain

This commit is contained in:
GTBarkley 2023-06-11 06:49:28 +00:00
parent 8b28694f0e
commit e65513322c

View file

@ -18,6 +18,14 @@ import Mathlib.Order.Height
variable {α : Type _} [Preorder α] (s : Set α) variable {α : Type _} [Preorder α] (s : Set α)
def finFun_to_list {n : } : (Fin n → α) → List α := by sorry
def series_to_chain : StrictSeries s → s.subchain
| ⟨length, toFun, strictMono⟩ =>
⟨ finFun_to_list (fun x => toFun x),
sorry⟩
-- there should be a coercion from WithTop to WithBot (WithTop ) but it doesn't seem to work -- there should be a coercion from WithTop to WithBot (WithTop ) but it doesn't seem to work
-- it looks like this might be because someone changed the instance from CoeCT to Coe during the port -- it looks like this might be because someone changed the instance from CoeCT to Coe during the port
lemma twoHeights : s ≠ ∅ → (some (Set.chainHeight s) : WithBot (WithTop )) = krullDim s := by lemma twoHeights : s ≠ ∅ → (some (Set.chainHeight s) : WithBot (WithTop )) = krullDim s := by