X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Fcontribs%2Fdama%2Fdama%2Fmodels%2Fq_value_skip.ma;h=e69de29bb2d1d6434b8b29ae775ad8c2e48c5391;hb=8d367045e504f594c280d2c87f906695ef9671ee;hp=e639582e1d7fc856baf39bdd67735b260b4d1d99;hpb=fa3ef782b1336310a78868e7dfc900fa988ee2ab;p=helm.git diff --git a/helm/software/matita/contribs/dama/dama/models/q_value_skip.ma b/helm/software/matita/contribs/dama/dama/models/q_value_skip.ma index e639582e1..e69de29bb 100644 --- a/helm/software/matita/contribs/dama/dama/models/q_value_skip.ma +++ b/helm/software/matita/contribs/dama/dama/models/q_value_skip.ma @@ -1,34 +0,0 @@ -(**************************************************************************) -(* ___ *) -(* ||M|| *) -(* ||A|| A project by Andrea Asperti *) -(* ||T|| *) -(* ||I|| Developers: *) -(* ||T|| The HELM team. *) -(* ||A|| http://helm.cs.unibo.it *) -(* \ / *) -(* \ / This file is distributed under the terms of the *) -(* v GNU General Public License Version 2 *) -(* *) -(**************************************************************************) - -include "models/q_shift.ma". - -lemma q_cmp2: - ∀a,b:ℚ.a < b ∨ b ≤ a. -intros; cases (q_cmp a b); -[1: right; apply q_eq_to_le; symmetry; assumption; -|2: left; assumption; -|3: right; apply q_lt_to_le; assumption;] -qed. - - - -lemma value_skip: - ∀f,i,b,tl. bars f = b::tl → start f + Qpos (\fst b) < i → - \fst (value f i) = \fst (value (mk_q_f (start f + Qpos (\fst b)) tl) i). -intros; cases (value f i); cases H2; clear H2; -[1: cases (?:False); apply (q_lt_corefl (start f)); cases H3; clear H3 H4 H5; - apply (q_lt_trans ???? H2); -|2: -simplify in ⊢ (? ? % ?);