Zulip Chat Archive
Stream: maths
Topic: graphs edge_finset
Shimon Cohen (Jun 06 2023 at 10:13):
What I need to add to make it work?
import combinatorics.simple_graph.basic
import data.fintype.basic
import data.fintype.card
import data.fintype.powerset
open fintype
variables {V : Type*} [fintype V] [decidable_eq V]
#check {gm : simple_graph V // card (gm.edge_set) = 5}
#check {gm : simple_graph V // card (gm.edge_finset) = 5}
Eric Wieser (Jun 06 2023 at 12:31):
Does this work?
#check {gm : simple_graph V // ∃ decidable_rel gm.adj, by exactI card (gm.edge_finset) = 5}
Eric Wieser (Jun 06 2023 at 12:32):
(docs#simple_graph.edge_finset)
Kyle Miller (Jun 06 2023 at 13:50):
There's also avoiding decidability:
variables {V : Type*} -- optional: [fintype V]
#check {gm : simple_graph V // nat.card gm.edge_set = 5}
What to choose depends on what you're trying to do with this type though.
Shimon Cohen (Jun 06 2023 at 15:34):
Eric Wieser said:
Does this work?
#check {gm : simple_graph V // ∃ decidable_rel gm.adj, by exactI card (gm.edge_finset) = 5}
No ): error: "invalid binder, atomic identifier expected"
Shimon Cohen (Jun 06 2023 at 15:36):
Kyle Miller said:
There's also avoiding decidability:
variables {V : Type*} -- optional: [fintype V] #check {gm : simple_graph V // nat.card gm.edge_set = 5}
What to choose depends on what you're trying to do with this type though.
where nat.card is defined?
Kyle Miller (Jun 06 2023 at 16:07):
Shimon Cohen (Jun 06 2023 at 18:18):
nice, I will try to use it with hope that inifinity will not hunt me later ;)
Last updated: Dec 20 2023 at 11:08 UTC