Theory Ribbons_Interfaces
section ‹Ribbon proof interfaces›
theory Ribbons_Interfaces imports
Ribbons_Basic
Proofchain
"HOL-Library.FSet"
begin
text ‹Interfaces are the top and bottom boundaries through which diagrams
can be connected into a surrounding context. For instance, when composing two
diagrams vertically, the bottom interface of the upper diagram must match the
top interface of the lower diagram.
We define a datatype of concrete interfaces. We then quotient by the
associativity, commutativity and unity properties of our
horizontal-composition operator.›
subsection ‹Syntax of interfaces›