In this theory we consider properties of functions that are binary operations, that is they map \(X\times X\) into \(X\).
It happens quite often that we have a binary operation on some set and we need a similar operation that is defined for functions on that set. For example once we know how to add real numbers we also know how to add real-valued functions: for \(f,g:X \rightarrow \mathbf{R}\) we define \((f+g)(x) = f(x) + g(x)\). Note that formally the \(+\) means something different on the left hand side of this equality than on the right hand side. This section aims at formalizing this process. We will call it "lifting to a function space", if you have a suggestion for a better name, please let me know.
Since we are writing in generic set notation, the definition below is a bit complicated. Here it what it says: Given a set \(X\) and another set \(f\) (that represents a binary function on \(X\)) we are defining \(f\) lifted to function space over \(X\) as the binary function (a set of pairs) on the space \(F = X \rightarrow \textrm{range}(f)\) such that the value of this function on pair \(\langle a,b \rangle\) of functions on \(X\) is another function \(c\) on \(X\) with values defined by \(c(x) = f\langle a(x), b(x)\rangle\).
definition
\( f \text{ lifted to function space over } X \equiv \) \( \{\langle p,\{\langle x,f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \rangle .\ x \in X\}\rangle .\ \) \( p \in (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f))\} \)
The result of the lift belongs to the function space.
lemma func_ZF_1_L1:
assumes A1: \( f : Y\times Y\rightarrow Y \) and A2: \( p \in (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f)) \)
shows \( \{\langle x,f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \rangle .\ x \in X\} : X\rightarrow \text{range}(f) \)proofThe values of the lift are defined by the value of the liftee in a natural way.
lemma func_ZF_1_L2:
assumes A1: \( f : Y\times Y\rightarrow Y \) and A2: \( p \in (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f)) \) and A3: \( x\in X \) and A4: \( P = \{\langle x,f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \rangle .\ x \in X\} \)
shows \( P(x) = f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \)proofFunction lifted to a function space results in function space operator.
theorem func_ZF_1_L3:
assumes \( f : Y\times Y\rightarrow Y \) and \( F = f \text{ lifted to function space over } X \)
shows \( F : (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f))\rightarrow (X\rightarrow \text{range}(f)) \) using assms, Lift2FcnSpce_def, func_ZF_1_L1, ZF_fun_from_totalThe values of the lift are defined by the values of the liftee in the natural way.
theorem func_ZF_1_L4:
assumes A1: \( f : Y\times Y\rightarrow Y \) and A2: \( F = f \text{ lifted to function space over } X \) and A3: \( s:X\rightarrow \text{range}(f) \), \( r:X\rightarrow \text{range}(f) \) and A4: \( x\in X \)
shows \( (F\langle s,r\rangle )(x) = f\langle s(x),r(x)\rangle \)proofIn this section we define associative and commutative operations and prove that they remain such when we lift them to a function space.
Typically we say that a binary operation "\(\cdot \)" on a set \(G\) is ''associative'' if \((x\cdot y)\cdot z = x\cdot (y\cdot z)\) for all \(x,y,z \in G\). Our actual definition below does not use the multiplicative notation so that we can apply it equally to the additive notation \(+\) or whatever infix symbol we may want to use. Instead, we use the generic set theory notation and write \(P\langle x,y \rangle\) to denote the value of the operation \(P\) on a pair \(\langle x,y \rangle \in G\times G\).
definition
\( P \text{ is associative on } G \equiv P : G\times G\rightarrow G \wedge \) \( (\forall x \in G.\ \forall y \in G.\ \forall z \in G.\ \) \( ( P(\langle P(\langle x,y\rangle ),z\rangle ) = P( \langle x,P(\langle y,z\rangle )\rangle ))) \)
A binary function \(f: X\times X \rightarrow Y\) is commutative if \(f\langle x,y \rangle = f\langle y,x \rangle\). Note that in the definition of associativity above we talk about binary ''operation'' and here we say use the term binary ''function''. This is not set in stone, but usually the word "operation" is used when the range is a factor of the domain, while the word "function" allows the range to be a completely unrelated set.
definition
\( f \text{ is commutative on } G \equiv \forall x\in G.\ \forall y\in G.\ f\langle x,y\rangle = f\langle y,x\rangle \)
The lift of a commutative function is commutative.
lemma func_ZF_2_L1:
assumes A1: \( f : G\times G\rightarrow G \) and A2: \( F = f \text{ lifted to function space over } X \) and A3: \( s : X\rightarrow \text{range}(f) \), \( r : X\rightarrow \text{range}(f) \) and A4: \( f \text{ is commutative on } G \)
shows \( F\langle s,r\rangle = F\langle r,s\rangle \)proofThe lift of a commutative function is commutative on the function space.
lemma func_ZF_2_L2:
assumes \( f : G\times G\rightarrow G \) and \( f \text{ is commutative on } G \) and \( F = f \text{ lifted to function space over } X \)
shows \( F \text{ is commutative on } (X\rightarrow \text{range}(f)) \) using assms, IsCommutative_def, func_ZF_2_L1The lift of an associative function is associative.
lemma func_ZF_2_L3:
assumes A2: \( F = f \text{ lifted to function space over } X \) and A3: \( s : X\rightarrow \text{range}(f) \), \( r : X\rightarrow \text{range}(f) \), \( q : X\rightarrow \text{range}(f) \) and A4: \( f \text{ is associative on } G \)
shows \( F\langle F\langle s,r\rangle ,q\rangle = F\langle s,F\langle r,q\rangle \rangle \)proofThe lift of an associative function is associative on the function space.
lemma func_ZF_2_L4:
assumes A1: \( f \text{ is associative on } G \) and A2: \( F = f \text{ lifted to function space over } X \)
shows \( F \text{ is associative on } (X\rightarrow \text{range}(f)) \)proofIn this section we consider conditions under which restriction of the operation to a set inherits properties like commutativity and associativity.
The commutativity is inherited when restricting a function to a set.
lemma func_ZF_4_L1:
assumes A1: \( f:X\times X\rightarrow Y \) and A2: \( A\subseteq X \) and A3: \( f \text{ is commutative on } X \)
shows \( \text{restrict}(f,A\times A) \text{ is commutative on } A \)proofNext we define what it means that a set is closed with respect to an operation.
definition
\( A \text{ is closed under } f \equiv \forall x\in A.\ \forall y\in A.\ f\langle x,y\rangle \in A \)
Associative operation restricted to a set that is closed with resp. to this operation is associative.
lemma func_ZF_4_L2:
assumes A1: \( f \text{ is associative on } X \) and A2: \( A\subseteq X \) and A3: \( A \text{ is closed under } f \) and A4: \( x\in A \), \( y\in A \), \( z\in A \) and A5: \( g = \text{restrict}(f,A\times A) \)
shows \( g\langle g\langle x,y\rangle ,z\rangle = g\langle x,g\langle y,z\rangle \rangle \)proofAn associative operation restricted to a set that is closed with resp. to this operation is associative on the set.
lemma func_ZF_4_L3:
assumes A1: \( f \text{ is associative on } X \) and A2: \( A\subseteq X \) and A3: \( A \text{ is closed under } f \)
shows \( \text{restrict}(f,A\times A) \text{ is associative on } A \)proofThe essential condition to show that if a set \(A\) is closed with respect to an operation, then it is closed under this operation restricted to any superset of \(A\).
lemma func_ZF_4_L4:
assumes \( A \text{ is closed under } f \) and \( A\subseteq B \) and \( x\in A \), \( y\in A \) and \( g = \text{restrict}(f,B\times B) \)
shows \( g\langle x,y\rangle \in A \) using assms, IsOpClosed_def, restrictIf a set \(A\) is closed under an operation, then it is closed under this operation restricted to any superset of \(A\).
lemma func_ZF_4_L5:
assumes A1: \( A \text{ is closed under } f \) and A2: \( A\subseteq B \)
shows \( A \text{ is closed under } \text{restrict}(f,B\times B) \)proofThe essential condition to show that intersection of sets that are closed with respect to an operation is closed with respect to the operation.
lemma func_ZF_4_L6:
assumes \( A \text{ is closed under } f \) and \( B \text{ is closed under } f \) and \( x \in A\cap B \), \( y\in A\cap B \)
shows \( f\langle x,y\rangle \in A\cap B \) using assms, IsOpClosed_defIntersection of sets that are closed with respect to an operation is closed under the operation.
lemma func_ZF_4_L7:
assumes \( A \text{ is closed under } f \), \( B \text{ is closed under } f \)
shows \( A\cap B \text{ is closed under } f \) using assms, IsOpClosed_defFor any set \(X\) we can consider a binary operation on the set of functions \(f:X\rightarrow X\) defined by \(C(f,g) = f\circ g\). Composition of functions (or relations) is defined in the standard Isabelle distribution as a higher order function and denoted with the letter O. In this section we consider the corresponding two-argument ZF-function (binary operation), that is a subset of \(((X\rightarrow X)\times (X\rightarrow X))\times (X\rightarrow X)\).
We define the notion of composition on the set \(X\) as the binary operation on the function space \(X\rightarrow X\) that takes two functions and creates the their composition.
definition
\( \text{Composition}(X) \equiv \) \( \{\langle p,\text{fst}(p)\circ \text{snd}(p)\rangle .\ p \in (X\rightarrow X)\times (X\rightarrow X)\} \)
Composition operation is a function that maps \((X\rightarrow X)\times (X\rightarrow X)\) into \(X\rightarrow X\).
lemma func_ZF_5_L1:
shows \( \text{Composition}(X) : (X\rightarrow X)\times (X\rightarrow X)\rightarrow (X\rightarrow X) \) using comp_fun, Composition_def, ZF_fun_from_totalThe value of the composition operation is the composition of arguments.
lemma func_ZF_5_L2:
assumes \( f:X\rightarrow X \) and \( g:X\rightarrow X \)
shows \( \text{Composition}(X)\langle f,g\rangle = f\circ g \)proofWhat is the value of a composition on an argument?
lemma func_ZF_5_L3:
assumes \( f:X\rightarrow X \) and \( g:X\rightarrow X \) and \( x\in X \)
shows \( ( \text{Composition}(X)\langle f,g\rangle )(x) = f(g(x)) \) using assms, func_ZF_5_L2, comp_fun_applyThe essential condition to show that composition is associative.
lemma func_ZF_5_L4:
assumes A1: \( f:X\rightarrow X \), \( g:X\rightarrow X \), \( h:X\rightarrow X \) and A2: \( C = \text{Composition}(X) \)
shows \( C\langle C\langle f,g\rangle ,h\rangle = C\langle f,C\langle g,h\rangle \rangle \)proofComposition is an associative operation on \(X\rightarrow X\) (the space of functions that map \(X\) into itself).
lemma func_ZF_5_L5:
shows \( \text{Composition}(X) \text{ is associative on } (X\rightarrow X) \)proofIn this section we show some additional facts about the identity function defined in the standard Isabelle's Perm theory. Note there is also image_id_same lemma in func1 theory.
A function that maps every point to itself is the identity on its domain.
lemma indentity_fun:
assumes A1: \( f:X\rightarrow Y \) and A2: \( \forall x\in X.\ f(x)=x \)
shows \( f = id(X) \)proofComposing a function with identity does not change the function.
lemma func_ZF_6_L1A:
assumes A1: \( f : X\rightarrow X \)
shows \( \text{Composition}(X)\langle f,id(X)\rangle = f \), \( \text{Composition}(X)\langle id(X),f\rangle = f \)proofAn intuitively clear, but surprisingly nontrivial fact: identity is the only function from a singleton to itself.
lemma singleton_fun_id:
shows \( (\{x\} \rightarrow \{x\}) = \{id(\{x\})\} \)proofAnother trivial fact: identity is the only bijection of a singleton with itself.
lemma single_bij_id:
shows \( \text{bij}(\{x\},\{x\}) = \{id(\{x\})\} \)proofA kind of induction for the identity: if a function \(f\) is the identity on a set with a fixpoint of \(f\) removed, then it is the indentity on the whole set.
lemma id_fixpoint_rem:
assumes A1: \( f:X\rightarrow X \) and A2: \( p\in X \) and A3: \( f(p) = p \) and A4: \( \text{restrict}(f, X-\{p\}) = id(X-\{p\}) \)
shows \( f = id(X) \)proofSuppose we have a binary operation \(f : X \times X \rightarrow X\) written additively as \(f\langle x,y\rangle = x + y\). Such operation naturally defines another binary operation on the subsets of \(X\) that satisfies \(A+B = \{ x+y : x \in A, y\in B\}\). This new operation which we will call "\(f\) lifted to subsets" inherits many properties of \(f\), such as associativity, commutativity and existence of the neutral element. This notion is useful for considering interval arithmetics.
The next definition describes the notion of a binary operation lifted to subsets. It is written in a way that might be a bit unexpected, but really it is the same as the intuitive definition, but shorter. In the definition we take a pair \(p \in Pow(X)\times Pow(X)\), say \(p = \langle A, B\rangle \), where \(A,B \subseteq X\). Then we assign this pair of sets the set \(\{f\langle x,y \rangle : x\in A, y\in B \} = \{ f(x'): x' \in A\times B\}\) The set on the right hand side is the same as the image of \(A\times B\) under \(f\). In the definition we don't use \(A\) and \(B\) symbols, but write \( \text{fst}(p) \) and \( \text{snd}(p) \), resp. Recall that in Isabelle/ZF \( \text{fst}(p) \) and \( \text{snd}(p) \) denote the first and second components of an ordered pair \(p\). See the lemma lift_subsets_explained for a more intuitive notation.
definition
\( f \text{ lifted to subsets of } X \equiv \) \( \{\langle p, f(\text{fst}(p)\times \text{snd}(p))\rangle .\ p \in Pow(X)\times Pow(X)\} \)
The lift to subsets defines a binary operation on the subsets.
lemma lift_subsets_binop:
assumes A1: \( f : X \times X \rightarrow Y \)
shows \( (f \text{ lifted to subsets of } X) : Pow(X) \times Pow(X) \rightarrow Pow(Y) \)proofThe definition of the lift to subsets rewritten in a more intuitive notation. We would like to write the last assertion as \( F\langle A,B\rangle = \{f\langle x,y\rangle .\ x \in A, y \in B\} \), but Isabelle/ZF does not allow such syntax.
lemma lift_subsets_explained:
assumes A1: \( f : X\times X \rightarrow Y \) and A2: \( A \subseteq X \), \( B \subseteq X \) and A3: \( F = f \text{ lifted to subsets of } X \)
shows \( F\langle A,B\rangle \subseteq Y \) and \( F\langle A,B\rangle = f(A\times B) \), \( F\langle A,B\rangle = \{f(p).\ p \in A\times B\} \), \( F\langle A,B\rangle = \{f\langle x,y\rangle .\ \langle x,y\rangle \in A\times B\} \)proofA sufficient condition for a point to belong to a result of lifting to subsets.
lemma lift_subset_suff:
assumes A1: \( f : X \times X \rightarrow Y \) and A2: \( A \subseteq X \), \( B \subseteq X \) and A3: \( x\in A \), \( y\in B \) and A4: \( F = f \text{ lifted to subsets of } X \)
shows \( f\langle x,y\rangle \in F\langle A,B\rangle \)proofA kind of converse of lift_subset_apply, providing a necessary condition for a point to be in the result of lifting to subsets.
lemma lift_subset_nec:
assumes A1: \( f : X \times X \rightarrow Y \) and A2: \( A \subseteq X \), \( B \subseteq X \) and A3: \( F = f \text{ lifted to subsets of } X \) and A4: \( z \in F\langle A,B\rangle \)
shows \( \exists x y.\ x\in A \wedge y\in B \wedge z = f\langle x,y\rangle \)proofLifting to subsets inherits commutativity.
lemma lift_subset_comm:
assumes A1: \( f : X \times X \rightarrow Y \) and A2: \( f \text{ is commutative on } X \) and A3: \( F = f \text{ lifted to subsets of } X \)
shows \( F \text{ is commutative on } Pow(X) \)proofLifting to subsets inherits associativity. To show that \(F\langle \langle A,B\rangle C\rangle = F\langle A,F\langle B,C\rangle\rangle\) we prove two inclusions and the proof of the second inclusion is very similar to the proof of the first one.
lemma lift_subset_assoc:
assumes A1: \( f \text{ is associative on } X \) and A2: \( F = f \text{ lifted to subsets of } X \)
shows \( F \text{ is associative on } Pow(X) \)proofIn this section we deal with pairs of operations such that one is distributive with respect to the other, that is \(a\cdot (b+c) = a\cdot b + a\cdot c\) and \((b+c)\cdot a = b\cdot a + c\cdot a\). We show that this property is preserved under restriction to a set closed with respect to both operations. In EquivClass1 theory we show that this property is preserved by projections to the quotient space if both operations are congruent with respect to the equivalence relation.
We define distributivity as a statement about three sets. The first set is the set on which the operations act. The second set is the additive operation (a ZF function) and the third is the multiplicative operation.
definition
\( \text{IsDistributive}(X,A,M) \equiv (\forall a\in X.\ \forall b\in X.\ \forall c\in X.\ \) \( M\langle a,A\langle b,c\rangle \rangle = A\langle M\langle a,b\rangle ,M\langle a,c\rangle \rangle \wedge \) \( M\langle A\langle b,c\rangle ,a\rangle = A\langle M\langle b,a\rangle ,M\langle c,a\rangle \rangle ) \)
The essential condition to show that distributivity is preserved by restrictions to sets that are closed with respect to both operations.
lemma func_ZF_7_L1:
assumes A1: \( \text{IsDistributive}(X,A,M) \) and A2: \( Y\subseteq X \) and A3: \( Y \text{ is closed under } A \), \( Y \text{ is closed under } M \) and A4: \( A_r = \text{restrict}(A,Y\times Y) \), \( M_r = \text{restrict}(M,Y\times Y) \) and A5: \( a\in Y \), \( b\in Y \), \( c\in Y \)
shows \( M_r\langle a,A_r\langle b,c\rangle \rangle = A_r\langle M_r\langle a,b\rangle ,M_r\langle a,c\rangle \rangle \wedge \) \( M_r\langle A_r\langle b,c\rangle ,a \rangle = A_r\langle M_r\langle b,a\rangle , M_r\langle c,a\rangle \rangle \)proofDistributivity is preserved by restrictions to sets that are closed with respect to both operations.
lemma func_ZF_7_L2:
assumes \( \text{IsDistributive}(X,A,M) \) and \( Y\subseteq X \) and \( Y \text{ is closed under } A \), \( Y \text{ is closed under } M \) and \( A_r = \text{restrict}(A,Y\times Y) \), \( M_r = \text{restrict}(M,Y\times Y) \)
shows \( \text{IsDistributive}(Y,A_r,M_r) \)proofassumes \( f:X\rightarrow Y \)
shows \( \text{range}(f) \subseteq Y \)assumes \( \forall x\in X.\ b(x) \in Y \)
shows \( \{\langle x,b(x)\rangle .\ x\in X\} : X\rightarrow Y \)assumes \( f : Y\times Y\rightarrow Y \) and \( p \in (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f)) \)
shows \( \{\langle x,f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \rangle .\ x \in X\} : X\rightarrow \text{range}(f) \)assumes \( f:X\rightarrow Y \), \( x\in X \) and \( f = \{\langle x,b(x)\rangle .\ x\in X\} \)
shows \( f(x) = b(x) \) and \( b(x)\in Y \)assumes \( f : Y\times Y\rightarrow Y \) and \( p \in (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f)) \) and \( x\in X \) and \( P = \{\langle x,f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \rangle .\ x \in X\} \)
shows \( P(x) = f\langle \text{fst}(p)(x),\text{snd}(p)(x)\rangle \)assumes \( f : Y\times Y\rightarrow Y \) and \( F = f \text{ lifted to function space over } X \)
shows \( F : (X\rightarrow \text{range}(f))\times (X\rightarrow \text{range}(f))\rightarrow (X\rightarrow \text{range}(f)) \)assumes \( f : Y\times Y\rightarrow Y \) and \( F = f \text{ lifted to function space over } X \) and \( s:X\rightarrow \text{range}(f) \), \( r:X\rightarrow \text{range}(f) \) and \( x\in X \)
shows \( (F\langle s,r\rangle )(x) = f\langle s(x),r(x)\rangle \)assumes \( f : G\times G\rightarrow G \) and \( F = f \text{ lifted to function space over } X \) and \( s : X\rightarrow \text{range}(f) \), \( r : X\rightarrow \text{range}(f) \) and \( f \text{ is commutative on } G \)
shows \( F\langle s,r\rangle = F\langle r,s\rangle \)assumes \( F = f \text{ lifted to function space over } X \) and \( s : X\rightarrow \text{range}(f) \), \( r : X\rightarrow \text{range}(f) \), \( q : X\rightarrow \text{range}(f) \) and \( f \text{ is associative on } G \)
shows \( F\langle F\langle s,r\rangle ,q\rangle = F\langle s,F\langle r,q\rangle \rangle \)assumes \( f:X\rightarrow Y \) and \( A\subseteq X \) and \( \forall x\in A.\ f(x) \in Z \)
shows \( \text{restrict}(f,A) : A\rightarrow Z \)assumes \( f \text{ is associative on } X \) and \( A\subseteq X \) and \( A \text{ is closed under } f \) and \( x\in A \), \( y\in A \), \( z\in A \) and \( g = \text{restrict}(f,A\times A) \)
shows \( g\langle g\langle x,y\rangle ,z\rangle = g\langle x,g\langle y,z\rangle \rangle \)assumes \( A \text{ is closed under } f \) and \( A\subseteq B \) and \( x\in A \), \( y\in A \) and \( g = \text{restrict}(f,B\times B) \)
shows \( g\langle x,y\rangle \in A \)assumes \( f:X\rightarrow X \) and \( g:X\rightarrow X \)
shows \( \text{Composition}(X)\langle f,g\rangle = f\circ g \)assumes \( f:X\rightarrow X \) and \( g:X\rightarrow X \) and \( x\in X \)
shows \( ( \text{Composition}(X)\langle f,g\rangle )(x) = f(g(x)) \)assumes \( f:X\rightarrow X \), \( g:X\rightarrow X \), \( h:X\rightarrow X \) and \( C = \text{Composition}(X) \)
shows \( C\langle C\langle f,g\rangle ,h\rangle = C\langle f,C\langle g,h\rangle \rangle \)assumes \( f: X\rightarrow Y \), \( g: X\rightarrow Z \) and \( \forall x\in X.\ f(x) = g(x) \)
shows \( f = g \)assumes \( f:X\rightarrow Y \)
shows \( f(B) \subseteq \text{range}(f) \) and \( f(B) \subseteq Y \)assumes \( f : X \times X \rightarrow Y \)
shows \( (f \text{ lifted to subsets of } X) : Pow(X) \times Pow(X) \rightarrow Pow(Y) \)assumes \( f:X\rightarrow Y \) and \( A\subseteq X \)
shows \( f(A) = \{f(x).\ x \in A\} \)assumes \( \forall x\in X.\ \forall y\in Y.\ a(\langle x,y\rangle ) = b(x,y) \)
shows \( \{a(p).\ p \in X\times Y\} = \{b(x,y).\ \langle x,y\rangle \in X\times Y\} \)assumes \( f : X\times X \rightarrow Y \) and \( A \subseteq X \), \( B \subseteq X \) and \( F = f \text{ lifted to subsets of } X \)
shows \( F\langle A,B\rangle \subseteq Y \) and \( F\langle A,B\rangle = f(A\times B) \), \( F\langle A,B\rangle = \{f(p).\ p \in A\times B\} \), \( F\langle A,B\rangle = \{f\langle x,y\rangle .\ \langle x,y\rangle \in A\times B\} \)assumes \( f : X \times X \rightarrow Y \) and \( A \subseteq X \), \( B \subseteq X \) and \( F = f \text{ lifted to subsets of } X \) and \( z \in F\langle A,B\rangle \)
shows \( \exists x y.\ x\in A \wedge y\in B \wedge z = f\langle x,y\rangle \)assumes \( f : X \times X \rightarrow Y \) and \( A \subseteq X \), \( B \subseteq X \) and \( x\in A \), \( y\in B \) and \( F = f \text{ lifted to subsets of } X \)
shows \( f\langle x,y\rangle \in F\langle A,B\rangle \)assumes \( \text{IsDistributive}(X,A,M) \) and \( Y\subseteq X \) and \( Y \text{ is closed under } A \), \( Y \text{ is closed under } M \) and \( A_r = \text{restrict}(A,Y\times Y) \), \( M_r = \text{restrict}(M,Y\times Y) \) and \( a\in Y \), \( b\in Y \), \( c\in Y \)
shows \( M_r\langle a,A_r\langle b,c\rangle \rangle = A_r\langle M_r\langle a,b\rangle ,M_r\langle a,c\rangle \rangle \wedge \) \( M_r\langle A_r\langle b,c\rangle ,a \rangle = A_r\langle M_r\langle b,a\rangle , M_r\langle c,a\rangle \rangle \)