]> matita.cs.unibo.it Git - helm.git/blob - matita/matita/contribs/lambda-delta/Basic-2/substitution/tps_split.ma
8d093e46bf58e14e7f5ffbeb4fc35835e4431185
[helm.git] / matita / matita / contribs / lambda-delta / Basic-2 / substitution / tps_split.ma
1 (*
2     ||M||  This file is part of HELM, an Hypertextual, Electronic
3     ||A||  Library of Mathematics, developed at the Computer Science
4     ||T||  Department of the University of Bologna, Italy.
5     ||I||
6     ||T||
7     ||A||  This file is distributed under the terms of the
8     \   /  GNU General Public License Version 2
9      \ /
10       V_______________________________________________________________ *)
11
12 include "Basic-2/substitution/tps_lift.ma".
13
14 (* PARTIAL SUBSTITUTION ON TERMS ********************************************)
15
16 (* Split properties *********************************************************)
17
18 lemma tps_split_up: ∀L,T1,T2,d,e. L ⊢ T1 [d, e] ≫ T2 → ∀i. d ≤ i → i ≤ d + e →
19                     ∃∃T. L ⊢ T1 [d, i - d] ≫ T & L ⊢ T [i, d + e - i] ≫ T2.
20 #L #T1 #T2 #d #e #H elim H -L T1 T2 d e
21 [ /2/
22 | /2/
23 | #L #K #V #V1 #V2 #i #d #e #Hdi #Hide #HLK #HV1 #HV12 #IHV12 #j #Hdj #Hjde
24   elim (lt_or_ge i j) #Hij
25   [ -HV1 Hide;
26     lapply (drop_fwd_drop2 … HLK) #HLK'
27     elim (IHV12 (j - i - 1) ? ?) -IHV12; normalize /2/ -Hjde <minus_n_O >arith_b2 // #W1 #HVW1 #HWV1
28     generalize in match HVW1 generalize in match Hij -HVW1 (**) (* rewriting in the premises, rewrites in the goal too *)
29     >(plus_minus_m_m_comm … Hdj) in ⊢ (% → % → ?) -Hdj #Hij' #HVW1
30     elim (lift_total W1 0 (i + 1)) #W2 #HW12
31     lapply (tps_lift_ge … HWV1 … HLK' HW12 HV12 ?) -HWV1 HLK' HV12 // >arith_a2 /3 width=6/
32   | -IHV12 Hdi Hdj;
33     generalize in match HV1 generalize in match Hide -HV1 Hide (**) (* rewriting in the premises, rewrites in the goal too *)
34     >(plus_minus_m_m_comm … Hjde) in ⊢ (% → % → ?) -Hjde #Hide #HV1
35     @ex2_1_intro [2: @tps_lref |1: skip | /2 width=6/ ] (**) (* /3 width=6 is too slow *)
36   ]
37 | #L #I #V1 #V2 #T1 #T2 #d #e #_ #_ #IHV12 #IHT12 #i #Hdi #Hide
38   elim (IHV12 i ? ?) -IHV12 // #V #HV1 #HV2
39   elim (IHT12 (i + 1) ? ?) -IHT12 [2: /2 by arith4/ |3: /2/ ] (* just /2/ is too slow *)
40   -Hdi Hide >arith_c1 >arith_c1x #T #HT1 #HT2
41   @ex2_1_intro [2,3: @tps_bind | skip ] (**) (* explicit constructors *)
42   [3: @HV1 |4: @HT1 |5: // |1,2: skip | /3 width=5/ ]
43 | #L #I #V1 #V2 #T1 #T2 #d #e #_ #_ #IHV12 #IHT12 #i #Hdi #Hide
44   elim (IHV12 i ? ?) -IHV12 // elim (IHT12 i ? ?) -IHT12 //
45   -Hdi Hide /3 width=5/
46 ]
47 qed.
48
49 lemma tps_inv_lift1_up: ∀L,U1,U2,dt,et. L ⊢ U1 [dt, et] ≫ U2 →
50                         ∀K,d,e. ↓[d, e] L ≡ K → ∀T1. ↑[d, e] T1 ≡ U1 →
51                         d ≤ dt → dt ≤ d + e → d + e ≤ dt + et →
52                         ∃∃T2. K ⊢ T1 [d, dt + et - (d + e)] ≫ T2 & ↑[d, e] T2 ≡ U2.
53 #L #U1 #U2 #dt #et #HU12 #K #d #e #HLK #T1 #HTU1 #Hddt #Hdtde #Hdedet
54 elim (tps_split_up … HU12 (d + e) ? ?) -HU12 // -Hdedet #U #HU1 #HU2
55 lapply (tps_weak … HU1 d e ? ?) -HU1 // <plus_minus_m_m_comm // -Hddt Hdtde #HU1
56 lapply (tps_inv_lift1_eq … HU1 … HTU1) -HU1 #HU1 destruct -U1;
57 elim (tps_inv_lift1_ge … HU2 … HLK … HTU1 ?) -HU2 HLK HTU1 // <minus_plus_m_m /2/
58 qed.