Theory Bool_Func
section‹Boolean functions›
theory Bool_Func
imports Main
begin
text‹
The end result of our implementation is verified against these functions:
›
type_synonym 'a boolfunc = "('a ⇒ bool) ⇒ bool"
text‹if-then-else on boolean functions.›
definition "bf_ite i t e ≡ (λl. if i l then t l else e l)"
text‹if-then-else is interesting because we can, together with constant true and false, represent all binary boolean functions using maximally two applications of it.›
abbreviation "bf_True ≡ (λl. True)"
abbreviation "bf_False ≡ (λl. False)"
text‹A quick demonstration:›
definition "bf_and a b ≡ bf_ite a b bf_False"
lemma "(bf_and a b) as ⟷ a as ∧ b as" unfolding bf_and_def bf_ite_def by meson
definition "bf_not b ≡ bf_ite b bf_False bf_True"
lemma bf_not_alt: "bf_not a as ⟷ ¬a as" unfolding bf_not_def bf_ite_def by meson
text‹For convenience, we want a few functions more:›
definition "bf_or a b ≡ bf_ite a bf_True b"
definition "bf_lit v ≡ (λl. l v)"
definition "bf_if v t e ≡ bf_ite (bf_lit v) t e"
lemma bf_if_alt: "bf_if v t e = (λl. if l v then t l else e l)" unfolding bf_if_def bf_ite_def bf_lit_def ..
definition "bf_nand a b = bf_not (bf_and a b)"
definition "bf_nor a b = bf_not (bf_or a b)"
definition "bf_biimp a b = (bf_ite a b (bf_not b))"
lemma bf_biimp_alt: "bf_biimp a b = (λl. a l ⟷ b l)" unfolding bf_biimp_def bf_not_def bf_ite_def by(simp add: fun_eq_iff)
definition "bf_xor a b = bf_not (bf_biimp a b)"
lemma bf_xor_alt: "bf_xor a b = (bf_ite a (bf_not b) b)"
unfolding bf_xor_def bf_biimp_def bf_not_def
unfolding bf_ite_def
by simp
text‹All of these are implemented and had their implementation verified.›
definition "bf_imp a b = bf_ite a b bf_True"
lemma bf_imp_alt: "bf_imp a b = bf_or (bf_not a) b" unfolding bf_or_def bf_not_def bf_imp_def unfolding bf_ite_def unfolding fun_eq_iff by simp
lemma [dest!,elim!]: "bf_False = bf_True ⟹ False" "bf_True = bf_False ⟹ False" unfolding fun_eq_iff by simp_all
lemmas [simp] = bf_and_def bf_or_def bf_nand_def bf_biimp_def bf_xor_alt bf_nor_def bf_not_def
subsection‹Shannon decomposition›
text‹
A restriction of a boolean function on a variable is creating the boolean function that evaluates as if that variable was set to a fixed value:
›
definition "bf_restrict (i::'a) (val::bool) (f::'a boolfunc) ≡ (λv. f (v(i:=val)))"
text ‹
Restrictions are useful, because they remove variables from the set of significant variables:
›
definition "bf_vars bf = {v. ∃as. bf_restrict v True bf as ≠ bf_restrict v False bf as}"
lemma "var ∉ bf_vars (bf_restrict var val ex)"
unfolding bf_vars_def bf_restrict_def by(simp)
text‹
We can decompose calculating if-then-else into computing if-then-else of two triples of functions with one variable restricted to true / false.
Given that the functions have finite arity, we can use this to construct a recursive definition.
›
lemma brace90shannon: "bf_ite F G H ass =
bf_ite (λl. l i)
(bf_ite (bf_restrict i True F) (bf_restrict i True G) (bf_restrict i True H))
(bf_ite (bf_restrict i False F) (bf_restrict i False G) (bf_restrict i False H)) ass"
unfolding bf_ite_def bf_restrict_def by (auto simp add: fun_upd_idem)
end