mirror of
https://github.com/GTBarkley/comm_alg.git
synced 2024-12-26 07:38:36 -06:00
function relating the offbrand notions of chain
This commit is contained in:
parent
8b28694f0e
commit
e65513322c
1 changed files with 8 additions and 0 deletions
|
@ -18,6 +18,14 @@ import Mathlib.Order.Height
|
|||
|
||||
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
|
||||
-- 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
|
||||
|
|
Loading…
Reference in a new issue