From: Wilmer Ricciotti <ricciott@cs.unibo.it> Date: Wed, 16 Jan 2013 16:01:54 +0000 (+0000) Subject: added null character to the alphabet X-Git-Tag: make_still_working~1340 X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=commitdiff_plain;h=e47584d3cc500acd8ffb533810daabd3b2ff8300;p=helm.git added null character to the alphabet --- diff --git a/matita/matita/lib/turing/multi_universal/alphabet.ma b/matita/matita/lib/turing/multi_universal/alphabet.ma index deb1dceec..8a6859669 100644 --- a/matita/matita/lib/turing/multi_universal/alphabet.ma +++ b/matita/matita/lib/turing/multi_universal/alphabet.ma @@ -15,33 +15,36 @@ include "basics/finset.ma". inductive unialpha : Type[0] â -| bit : bool â unialpha -| bar : unialpha. +| bit : bool â unialpha +| null : unialpha +| bar : unialpha. definition unialpha_eq â λa1,a2.match a1 with [ bit x â match a2 with [ bit y â ¬ xorb x y | _ â false ] - | bar â match a2 with [ bar â true | _ â false ] ]. + | bar â match a2 with [ bar â true | _ â false ] + | null â match a2 with [ null â true | _ â false ] ]. definition DeqUnialpha â mk_DeqSet unialpha unialpha_eq ?. * [ #x * [ #y cases x cases y normalize % // #Hfalse destruct | *: normalize % #Hfalse destruct ] - | * [ #y ] normalize % #H1 destruct % ] + | *: * [1,4: #y ] normalize % #H1 destruct % ] qed. lemma unialpha_unique : - uniqueb DeqUnialpha [bit true;bit false;bar] = true. + uniqueb DeqUnialpha [bit true;bit false;null;bar] = true. // qed. lemma unialpha_complete :âx:DeqUnialpha. - memb ? x [bit true;bit false;bar] = true. + memb ? x [bit true;bit false;null;bar] = true. * // * // qed. definition FSUnialpha â - mk_FinSet DeqUnialpha [bit true;bit false;bar] + mk_FinSet DeqUnialpha [bit true;bit false;null;bar] unialpha_unique unialpha_complete. (*************************** testing characters *******************************) definition is_bit â λc.match c with [ bit _ â true | _ â false ]. -definition is_bar â λc.match c with [ bar â true | _ â false ]. \ No newline at end of file +definition is_bar â λc.match c with [ bar â true | _ â false ]. +definition is_null â λc.match c with [ null â true | _ â false ]. \ No newline at end of file