Zulip Chat Archive

Stream: Is there code for X?

Topic: Code for studying infinite rooted trees


Abraham Solomon (Nov 10 2024 at 06:36):

Hey all,

I have been trying to define some results for infinite rooted trees, I have some vague ideas of how to do it -- but curious if something already exists.

My goal is to define for an infinite rooted tree TT the notion of a cutset ΠT\Pi \subset T -- a finite subset of vertices such that every infinite path from the root has a non-empty intersection with Π\Pi.

I can define an infinite graph that's a tree, and currently working to adapt Mathlib.Combinatorics.SimpleGraph.Path to the infinite setting.

A very rough sketch is something like this(assuming the tree has no leaves other than the root):

import Mathlib.Combinatorics.SimpleGraph.Path

variable {V : Type u} (G : SimpleGraph V)

def IsAcyclic : Prop :=  v : V (c : G.Walk v v), ¬c.IsCycle

inductive Infinite_Walk : V  Type u
  | nil {u : V} : Infinite_Walk u
  | cons {u v: V} (h : G.Adj u v) (p : Infinite_Walk u) : Infinite_Walk v


def IsCutset (T: SimpleGraph V)(S: T.Subgraph)(h₁: T.Connected   IsAcyclic T) (root : V): Prop :=
  c : Infinite_Walk T root, (k : S.verts), (k  c)

Of course, to check membership is probably hard and requires some interoperability with finite paths. Does anyone know of anything like this?

The cardinality of all (unique) infinite paths is unfortunately often equal to the continuum, so there are complexities arising with that already; not to mention various other issues. But the above is just a rough idea.

Yaël Dillies (Nov 10 2024 at 09:33):

@Daniel Weber successfully implemented rooted trees as archimedean pred-orders (docs#PredOrder, docs#IsPredArchimedean). Could you reuse this idea?

Nir Paz (Nov 10 2024 at 09:39):

I'm not too familiar with these notions, is a tree with uncountable height an archimedean pred order? In set theory every ordinal is a tree (although I'm not sure if that's what @Abraham Solomon is going for here).

Nir Paz (Nov 10 2024 at 09:40):

Actually that's not a simple graph, so doesn't match the definition above

Abraham Solomon (Nov 10 2024 at 09:43):

Nir Paz said:

I'm not too familiar with these notions, is a tree with uncountable height an archimedean pred order? In set theory every ordinal is a tree (although I'm not sure if that's what Abraham Solomon is going for here).

I think that's the set theory type tree, which is connected to graph theory / rooted trees via Hasse diagrams -- but i want to be able to access the 'nth' level of an infinite walk.

Essentially, from the root, there exist degree(root) infinite paths at first (rays isomorphic to N\mathbb{N} with some darts(assume locally finite tree so degrees are all finite)).

Then, every time there is another child (since there are no leaves) this creates more rays inductively.

The easiest notion of cutset(s) for a tree TT with root ρ\rho are the level sets Sn:={vTv=n}S_{n} := \{ v \in T | |v| = n\} -- |\cdot| the graph distance from the root. If a tree TT is spherically symmetric ( something like the degree of vTv \in T depends only on v|v|) these are often all you need in practice not to lose generality.

Eventually, such notions allow the categorisation of all locally finite trees by their 'exponents', with more information for spherically symmetric trees. For example, for the perfect rooted infinite binary tree -- an exponent known as the branching number is 2; for d-ary trees this is d.

Abraham Solomon (Nov 10 2024 at 09:57):

Yaël Dillies said:

Daniel Weber successfully implemented rooted trees as archimedean pred-orders (docs#PredOrder, docs#IsPredArchimedean). Could you reuse this idea?

I think this could be similar to what i wanted, thanks!

I think the way it would be defined for me is for two vertices v,wTv,w \in T, vwv \leq w if both are on an infinite path together and vw|v| \leq |w|.

Daniel Weber (Nov 10 2024 at 10:20):

Nir Paz said:

I'm not too familiar with these notions, is a tree with uncountable height an archimedean pred order? In set theory every ordinal is a tree (although I'm not sure if that's what Abraham Solomon is going for here).

No, archimedeaness implies height ω\omega. A set theoretic tree is a partial order where every docs#Set.Iio is a well order, and then you can define the distance with docs#Ordinal.type (perhaps you can even relax the IsWellOrder in docs#Ordinal.typein to make it be the distance directly)

Daniel Weber (Nov 10 2024 at 10:24):

Abraham Solomon said:

Yaël Dillies said:

Daniel Weber successfully implemented rooted trees as archimedean pred-orders (docs#PredOrder, docs#IsPredArchimedean). Could you reuse this idea?

I think this could be similar to what i wanted, thanks!

I think the way it would be defined for me is for two vertices v,wTv,w \in T, vwv \leq w if both are on an infinite path together and vw|v| \leq |w|.

Maybe I misunderstand what you want to do, but can't you directly use docs#RootedTree and then define \left| \cdot \right| as Nat.find (bot_le (a := r)).exists_pred_iterate (this is also part of the definition of docs#IsPredArchimedean.findAtom, so it could be moved out of there)?

Abraham Solomon (Nov 10 2024 at 10:32):

Daniel Weber said:

Abraham Solomon said:

Yaël Dillies said:

Daniel Weber successfully implemented rooted trees as archimedean pred-orders (docs#PredOrder, docs#IsPredArchimedean). Could you reuse this idea?

I think this could be similar to what i wanted, thanks!

I think the way it would be defined for me is for two vertices v,wTv,w \in T, vwv \leq w if both are on an infinite path together and vw|v| \leq |w|.

Maybe I misunderstand what you want to do, but can't you directly use docs#RootedTree and then define \left| \cdot \right| as Nat.find (bot_le (a := r)).exists_pred_iterate (this is also part of the definition of docs#IsPredArchimedean.findAtom, so it could be moved out of there)?

Yea i think that could work, eventually i want to be able to define something like this:

inf{λ>0infΠzΠλz=0}\inf \{ \lambda > 0 | \inf_{\Pi}\sum_{z \in \Pi}\lambda^{-|z|} = 0\}.

Where the second infimum is taken over all cutsets of the tree TT; this is the branching number of the tree br(T)\text{br}(T) and for the binary tree is equal to 2(this is one of several exponents that can classify spherically symmetric trees). Almost by definition, it is larger than or equal to one.

With that as the end goal, ill have to be careful as to how the tree works with regards to its 'cutsets'.

The reference for doing this is from:
Russell Lyons and Yuval Peres. Probability on Trees and Networks. Cambridge
Series in Statistical and Probabilistic Mathematics. Cambridge University Press,
2017.

Daniel Weber (Nov 10 2024 at 10:42):

If I understood correctly, order theoretically a set Π\Pi is a cutset if for all xx there exists yΠy \in \Pi such that x,yx, y are comparable

Abraham Solomon (Nov 10 2024 at 10:44):

Daniel Weber said:

If I understood correctly, order theoretically a set Π\Pi is a cutset if for all xx there exists yΠy \in \Pi such that x,yx, y are comparable

Yea, and it must also be finite


Last updated: May 02 2025 at 03:31 UTC