-
Notifications
You must be signed in to change notification settings - Fork 298
feat(library): weak duality of max-flow min-cut theorem #18996
base: master
Are you sure you want to change the base?
Conversation
LaTeX is used.
Implemented in LaTeX
leanpkg.toml
Outdated
@@ -5,3 +5,4 @@ lean_version = "leanprover-community/lean:3.50.3" | |||
path = "src" | |||
|
|||
[dependencies] | |||
mathlib = {git = "https://github.com/leanprover-community/mathlib", rev = "290a7ba01fbcab1b64757bdaa270d28f4dcede35"} |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
This doesn't make any sense in mathlib itself!
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
Removed.
-- /-! | ||
-- Here is our second big lemma, if the active flow is maximum, | ||
-- then no augmenting path exists in the residual network. | ||
-- -/ | ||
|
||
-- lemma no_augm_path {V : Type*} [inst' : fintype V] | ||
-- (rsn : residual_network V) : (is_max_flow rsn.afn) -> no_augmenting_path rsn := | ||
-- begin |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
If this is intended to be part of a later PR, you should just delete it from this one.
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
Removed.
Max-Flow_Min-Cut_Proof.pdf
Outdated
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
This should either be:
- Hosted on your own website / arxiv, and linked from
references.bib
- Put in the module docstring, or in various smaller docstrings throughout the file. Note that the doc website supports LaTeX in
$$
s
(is_edge : V → V → Prop) | ||
(nonsymmetric : ∀ u v : V, ¬ ((is_edge u v) ∧ (is_edge v u))) | ||
|
||
structure capacity (V : Type*) [inst : fintype V] |
There was a problem hiding this comment.
Choose a reason for hiding this comment
The reason will be displayed to describe this comment to others. Learn more.
To me this looks like it would work better as
structure capacity (V : Type*) [inst : fintype V] | |
structure capacity {V : Type*} [inst : fintype V] (g : digraph V) |
Which says "a capacity on a particular graph". I assume you don't ever need to compare capacities between different graphs?
Formalise and validate the weak duality of the max-flow min-cut theorem, i.e. the value of every flow is less than or equal to the capacity of every cut.
The rest of the max-flow min-cut theorem proof is commented out because it contains sorry.