X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Fcontribs%2Fng_assembly%2Fcommon%2Fstring_lemmas.ma;h=be090076f0166fd3c0535010175f0fa7fcb11a70;hb=a90c31c1b53222bd6d57360c5ba5c2d0fe7d5207;hp=1b596170bbf0afbf5609db4d28ea8410d2c58d6d;hpb=4377e950998c9c63937582952a79975947aa9a45;p=helm.git diff --git a/helm/software/matita/contribs/ng_assembly/common/string_lemmas.ma b/helm/software/matita/contribs/ng_assembly/common/string_lemmas.ma index 1b596170b..be090076f 100755 --- a/helm/software/matita/contribs/ng_assembly/common/string_lemmas.ma +++ b/helm/software/matita/contribs/ng_assembly/common/string_lemmas.ma @@ -16,7 +16,7 @@ (* Progetto FreeScale *) (* *) (* Sviluppato da: Ing. Cosimo Oliboni, oliboni@cs.unibo.it *) -(* Sviluppo: 2008-2010 *) +(* Ultima modifica: 05/08/2009 *) (* *) (* ********************************************************************** *) @@ -30,17 +30,17 @@ include "common/list_utility_lemmas.ma". nlemma symmetric_eqstr : symmetricT (list ascii) bool eq_str. #s1; #s2; - napply (symmetric_bfoldrightlist2 ascii eq_ascii symmetric_eqascii s1 s2). + napply (symmetric_bfoldrightlist2 ascii eq_ascii s1 s2 symmetric_eqascii). nqed. nlemma eqstr_to_eq : ∀s,s'.eq_str s s' = true → s = s'. #s1; #s2; - napply (bfoldrightlist2_to_eq ascii eq_ascii eqascii_to_eq s1 s2). + napply (bfoldrightlist2_to_eq ascii eq_ascii s1 s2 eqascii_to_eq). nqed. nlemma eq_to_eqstr : ∀s,s'.s = s' → eq_str s s' = true. #s1; #s2; - napply (eq_to_bfoldrightlist2 ascii eq_ascii eq_to_eqascii s1 s2). + napply (eq_to_bfoldrightlist2 ascii eq_ascii s1 s2 eq_to_eqascii). nqed. nlemma decidable_str : ∀x,y:list ascii.decidable (x = y). @@ -50,13 +50,13 @@ nqed. nlemma neqstr_to_neq : ∀s,s'.eq_str s s' = false → s ≠ s'. #s1; #s2; - napply (nbfoldrightlist2_to_neq ascii eq_ascii ? s1 s2 …); + napply (nbfoldrightlist2_to_neq ascii eq_ascii s1 s2 …); napply neqascii_to_neq. nqed. nlemma neq_to_neqstr : ∀s,s'.s ≠ s' → eq_str s s' = false. #s1; #s2; - napply (neq_to_nbfoldrightlist2 ascii eq_ascii ?? s1 s2 …); + napply (neq_to_nbfoldrightlist2 ascii eq_ascii s1 s2 …); ##[ ##1: napply decidable_ascii ##| ##2: napply neq_to_neqascii ##] @@ -90,7 +90,7 @@ nlemma symmetric_eqstrid : symmetricT strId bool eq_strId. nrewrite > (symmetric_eqstr (str_elem si1) (str_elem si2)); nrewrite > (symmetric_eqnat (id_elem si1) (id_elem si2)); napply refl_eq. -nqed. +nqed. nlemma eqstrid_to_eq : ∀s,s'.eq_strId s s' = true → s = s'. #si1; #si2;