]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/turing/multi_to_mono/shift_trace.ma
component syntax_extensions was not declared
[helm.git] / matita / matita / lib / turing / multi_to_mono / shift_trace.ma
index 9ff88de28f7607db10cb60f43547774e70252103..1e5e36e9122050e5588c7c91f744dc1c2776daf5 100644 (file)
@@ -24,7 +24,7 @@ axiom regular_tail: ∀sig,n,l,i.
   regular_i sig n l i → regular_i sig n (tail ? l) i.
   
 axiom regular_extend: ∀sig,n,l,i.
-   regular_i sig n l i → regular_i sig n (l@[all_blank sig n]) i.
+   regular_i sig n l i → regular_i sig n (l@[all_blanks sig n]) i.
 
 axiom all_blank_after_blank: ∀sig,n,l1,b,l2,i. 
   nth i ? (vec … b) (blank ?) = blank ? → 
@@ -32,7 +32,7 @@ axiom all_blank_after_blank: ∀sig,n,l1,b,l2,i.
    
 lemma regular_trace_extl:  ∀sig,n,a,ls,rs,i.
   regular_trace sig n a ls rs i → 
-    regular_trace sig n a (ls@[all_blank sig n]) rs i.
+    regular_trace sig n a (ls@[all_blanks sig n]) rs i.
 #sig #n #a #ls #rs #i *
   [* #H1 #H2 % % // @(regular_extend … H1)
   |* #H1 #H2 %2 % // @(regular_extend … H1)
@@ -41,7 +41,7 @@ qed.
 
 lemma regular_cons_hd_rs: ∀sig,n.∀a:multi_sig sig n.∀ls,rs1,rs2,i.
   regular_trace sig n a ls (rs1@rs2) i → 
-    regular_trace sig n a ls (rs1@((hd ? rs2 (all_blank …))::(tail ? rs2))) i.
+    regular_trace sig n a ls (rs1@((hd ? rs2 (all_blanks …))::(tail ? rs2))) i.
 #sig #n #a #ls #rs1 #rs2 #i cases rs2 [2: #b #tl #H @H] 
 *[* #H1 >append_nil #H2 %1 % 
    [@H1 | whd in match (hd ???); @(regular_extend … rs1) //]
@@ -69,7 +69,7 @@ qed.
    improve semantics *)
    
 definition move_to_blank_L ≝ λsig,n,i.
-  (move_until ? L (no_blank sig n i)) · extend ? (all_blank sig n).
+  (move_until ? L (not_blank sig n i)) · extend ? (all_blanks sig n).
 
 (*
 definition R_move_to_blank_L ≝ λsig,n,i,t1,t2.
@@ -85,7 +85,7 @@ definition R_move_to_blank_L ≝ λsig,n,i,t1,t2.
 
 definition R_move_to_blank_L ≝ λsig,n,i,t1,t2.
 (current ? t1 = None ? → 
-  t2 = midtape (multi_sig sig n) (left ? t1) (all_blank …) (right ? t1)) ∧
+  t2 = midtape (multi_sig sig n) (left ? t1) (all_blanks …) (right ? t1)) ∧
 ∀ls,a,rs.
   t1 = midtape (multi_sig sig n) ls a rs → 
   regular_i sig n (a::ls) i →
@@ -93,17 +93,17 @@ definition R_move_to_blank_L ≝ λsig,n,i,t1,t2.
   (∃b,ls1,ls2.
     (regular_i sig n (ls1@b::ls2) i) ∧ 
     (∀j. j ≠ i → regular_trace … 
-      (hd ? (ls1@b::ls2) (all_blank …)) (tail ? (ls1@b::ls2)) rs j) ∧ 
-    (no_blank sig n i b = false) ∧ 
-    (hd (multi_sig sig n) (ls1@[b]) (all_blank …) = a) ∧ (* not implied by the next fact *)
-    (∀j.j n → to_blank_i ?? j (ls1@b::ls2) = to_blank_i ?? j (a::ls)) ∧
+      (hd ? (ls1@b::ls2) (all_blanks …)) (tail ? (ls1@b::ls2)) rs j) ∧ 
+    (not_blank sig n i b = false) ∧ 
+    (hd (multi_sig sig n) (ls1@[b]) (all_blanks …) = a) ∧ (* not implied by the next fact *)
+    (∀j.j n → to_blank_i ?? j (ls1@b::ls2) = to_blank_i ?? j (a::ls)) ∧
     t2 = midtape ? ls2 b ((reverse ? ls1)@rs)).
 
 theorem sem_move_to_blank_L: ∀sig,n,i. 
   move_to_blank_L sig n i  ⊨ R_move_to_blank_L sig n i.
 #sig #n #i 
 @(sem_seq_app ?????? 
-  (ssem_move_until_L ? (no_blank sig n i)) (sem_extend ? (all_blank sig n)))
+  (ssem_move_until_L ? (not_blank sig n i)) (sem_extend ? (all_blanks sig n)))
 #tin #tout * #t1 * * #Ht1a #Ht1b * #Ht2a #Ht2b %
   [#Hcur >(Ht1a Hcur) in Ht2a; /2 by /
   |#ls #a #rs #Htin #Hreg #Hreg2 -Ht1a cases (Ht1b … Htin)
@@ -122,11 +122,11 @@ theorem sem_move_to_blank_L: ∀sig,n,i.
       ]
     |* #b * #lss * * #H1 #H2 #Ht1 -Ht1b >Ht1 in Ht2a; 
      whd in match (left ??); whd in match (right ??); #Hout
-     %{(all_blank …)} %{(lss@[b])} %{[]}
+     %{(all_blanks …)} %{(lss@[b])} %{[]}
      %[%[%[%[%[<H2 @regular_extend // 
               |<H2 #j #jneqi whd in match (hd ???); whd in match (tail ??); 
                @regular_trace_extl @Hreg2 //]
-            |whd in match (no_blank ????); >blank_all_blank //]
+            |whd in match (not_blank ????); >blank_all_blanks //]
           |<H2 //]
         |#j #lejn <H2 @sym_eq @to_blank_i_ext]
       |>reverse_append >reverse_single @Hout normalize // 
@@ -138,9 +138,9 @@ qed.
 (******************************************************************************)
    
 definition shift_i_L ≝ λsig,n,i.
-   ncombf_r (multi_sig …) (shift_i sig n i) (all_blank sig n) ·
+   ncombf_r (multi_sig …) (shift_i sig n i) (all_blanks sig n) ·
    mti sig n i · 
-   extend ? (all_blank sig n).
+   extend ? (all_blanks sig n).
    
 definition R_shift_i_L ≝ λsig,n,i,t1,t2.
     (∀a,ls,rs. 
@@ -155,13 +155,13 @@ definition R_shift_i_L ≝ λsig,n,i,t1,t2.
         (∀x. mem ? x rs → nth i ? (vec … x) (blank ?) ≠ (blank ?)) ∧
         shift_l sig n i (a::rs) (rss@[b]) ∧
         t2 = midtape (multi_sig sig n) 
-          ((reverse ? (rss@[b]))@ls) (all_blank sig n) [ ]))).
+          ((reverse ? (rss@[b]))@ls) (all_blanks sig n) [ ]))).
 
 definition R_shift_i_L_new ≝ λsig,n,i,t1,t2.
   (∀a,ls,rs. 
    t1 = midtape ? ls a rs  → 
    ∃rs1,b,rs2,rss.
-      b = hd ? rs2 (all_blank sig n) ∧
+      b = hd ? rs2 (all_blanks sig n) ∧
       nth i ? (vec … b) (blank ?) = (blank ?) ∧
       rs = rs1@rs2 ∧ 
       (∀x. mem ? x rs1 → nth i ? (vec … x) (blank ?) ≠ (blank ?)) ∧
@@ -171,12 +171,12 @@ definition R_shift_i_L_new ≝ λsig,n,i,t1,t2.
 theorem sem_shift_i_L: ∀sig,n,i. shift_i_L sig n i  ⊨ R_shift_i_L sig n i.
 #sig #n #i 
 @(sem_seq_app ?????? 
-  (sem_ncombf_r (multi_sig sig n) (shift_i sig n i)(all_blank sig n))
+  (sem_ncombf_r (multi_sig sig n) (shift_i sig n i)(all_blanks sig n))
    (sem_seq ????? (ssem_mti sig n i) 
-    (sem_extend ? (all_blank sig n))))
+    (sem_extend ? (all_blanks sig n))))
 #tin #tout * #t1 * * #Ht1a #Ht1b * #t2 * * #Ht2a #Ht2b * #Htout1 #Htout2
 #a #ls #rs cases rs
-  [#Htin %2 %{(shift_i sig n i a (all_blank sig n))} %{[ ]} 
+  [#Htin %2 %{(shift_i sig n i a (all_blanks sig n))} %{[ ]} 
    %[%[#x @False_ind | @daemon]
     |lapply (Ht1a … Htin) -Ht1a -Ht1b #Ht1 
      lapply (Ht2a … Ht1) -Ht2a -Ht2b #Ht2 >Ht2 in Htout1; 
@@ -200,7 +200,7 @@ theorem sem_shift_i_L: ∀sig,n,i. shift_i_L sig n i  ⊨ R_shift_i_L sig n i.
       ]
     |* #b * #rss * * #H1 #H2 
      #Ht2 %2
-     %{(shift_i sig n i b (all_blank sig n))} %{(shift_i sig n i a a1::rss)}
+     %{(shift_i sig n i b (all_blanks sig n))} %{(shift_i sig n i a a1::rss)}
      %[%[@H1 |@daemon ]
       |>Ht2 in Htout1; #Htout >Htout //
        whd in match (left ??); whd in match (right ??);
@@ -221,53 +221,88 @@ theorem sem_shift_i_L_new: ∀sig,n,i.
    %{rs1} %{b} %{(b::rs2)} %{(a1::rss)} 
    %[%[%[%[%[//|@H2]|@H1]|@H3]|@H4] | whd in match (tail ??); @Ht2]
   |* #b * #rss * * #H1 #H2 #Ht2
-   %{rs} %{(all_blank sig n)} %{[]} %{(rss@[b])} 
-   %[%[%[%[%[//|@blank_all_blank]|//]|@H1]|@H2] | whd in match (tail ??); @Ht2]
+   %{rs} %{(all_blanks sig n)} %{[]} %{(rss@[b])} 
+   %[%[%[%[%[//|@blank_all_blanks]|//]|@H1]|@H2] | whd in match (tail ??); @Ht2]
   ]
 qed.
    
 
 (*******************************************************************************
-The following machine implements a full move of for a trace: we reach the left 
-border, shift the i-th trace and come back to the head position. *)  
+The following machine implements a full move for a trace: we reach the left 
+border, shift the i-th trace and come back to the head position. 
+The head may hold additional information A, so we suppose that the tape alphabet
+is the disjoint sum between A and the alphabet sig of the multi tape machine. *) 
+
+definition TA ≝ λA,sig. FinSum A sig.
+definition MTA ≝ λA,sig,n.multi_sig (TA A sig) n.
+
+definition is_head ≝ λA,sig.λc:sig_ext (TA A sig).
+  match c with
+  [ None ⇒ false
+  | Some a ⇒ match a with 
+     [ inl _ ⇒ true
+     | inr _ ⇒ false]].
+
+definition is_sig ≝ λA,sig.λc:sig_ext (TA A sig).
+  match c with
+  [ None ⇒ false
+  | Some a ⇒ match a with 
+     [ inl _ ⇒ false
+     | inr _ ⇒ true]].
+
+definition not_head ≝ λA,sig,n.λc:multi_sig (TA A sig) (S n).
+  ¬(is_head A sig (nth n ? (vec … c) (blank ?))).
+  
+lemma not_head_all_blanks : ∀A,sig,n. 
+  not_head A sig n (all_blanks … (S n)) = true.
+#A #sig #n whd in ⊢ (??%?); >blank_all_blanks //
+qed.  
+
+definition no_head_in ≝ λA,sig,n,l. 
+  ∀x. mem ? x (trace (TA A sig) (S n) n l) → is_head … x = false.
+
+(*
+lemma not_head_true: ∀A,sig,n,c. not_head A sig n c = true → 
+  is_head … (nth n ? (vec … c) (blank ?)) = false.
+*)
 
-(* this exclude the possibility that traces do not overlap: the head must 
-remain inside all traces *)
+lemma hd_nil : ∀A,d. hd A [ ] d = d. 
+// qed.
 
-definition mtiL ≝ λsig,n,i.
-   move_to_blank_L sig n i · 
-   shift_i_L sig n i ·
-   move_until ? L (no_head sig n). 
+definition mtiL ≝ λA,sig,n,i.
+   move_to_blank_L (TA A sig) (S n) i · 
+   shift_i_L (TA A sig) (S n) i ·
+   move_until ? L (not_head A sig n). 
    
-definition Rmtil ≝ λsig,n,i,t1,t2.
+definition Rmtil ≝ λA,sig,n,i,t1,t2.
   ∀ls,a,rs. 
-   t1 = midtape (multi_sig sig n) ls a rs → 
-   nth n ? (vec … a) (blank ?) = head ? →  
-   (∀i.regular_trace sig n a ls rs i) → 
+   t1 = midtape (MTA A sig (S n)) ls a rs → 
+   is_head A sig (nth n ? (vec … a) (blank ?)) = true →  
+   (∀i.regular_trace (TA A sig) (S n) a ls rs i) → 
    (* next: we cannot be on rightof on trace i *)
    (nth i ? (vec … a) (blank ?) = (blank ?) 
-     → nth i ? (vec … (hd ? rs (all_blank …))) (blank ?) ≠ (blank ?)) →
+     → nth i ? (vec … (hd ? rs (all_blanks …))) (blank ?) ≠ (blank ?)) →
    no_head_in … ls →   
    no_head_in … rs  → 
    (∃ls1,a1,rs1.
-     t2 = midtape (multi_sig …) ls1 a1 rs1 ∧
+     t2 = midtape (MTA A sig (S n)) ls1 a1 rs1 ∧
      (∀i.regular_trace … a1 ls1 rs1 i) ∧
-     (∀j. j ≤ n → j ≠ i → to_blank_i ? n j (a1::ls1) = to_blank_i ? n j (a::ls)) ∧
-     (∀j. j ≤ n → j ≠ i → to_blank_i ? n j rs1 = to_blank_i ? n j rs) ∧
-     (to_blank_i ? n i ls1 = to_blank_i ? n i (a::ls)) ∧
-     (to_blank_i ? n i (a1::rs1)) = to_blank_i ? n i rs).
+     (∀j. j ≤ n → j ≠ i → to_blank_i ? (S n) j (a1::ls1) = to_blank_i ? (S n) j (a::ls)) ∧
+     (∀j. j ≤ n → j ≠ i → to_blank_i ? (S n) j rs1 = to_blank_i ? (S n) j rs) ∧
+     (to_blank_i ? (S n) i ls1 = to_blank_i ? (S n) i (a::ls)) ∧
+     (to_blank_i ? (S n) i (a1::rs1)) = to_blank_i ? (S n) i rs).
 
-theorem sem_Rmtil: ∀sig,n,i. i < n → mtiL sig n i  ⊨ Rmtil sig n i.
-#sig #n #i #lt_in
+theorem sem_Rmtil: ∀A,sig,n,i. i < n → mtiL A sig n i  ⊨ Rmtil A sig n i.
+#A #sig #n #i #lt_in
 @(sem_seq_app ?????? 
   (sem_move_to_blank_L … )
    (sem_seq ????? (sem_shift_i_L_new …)
-    (ssem_move_until_L ? (no_head sig n))))
+    (ssem_move_until_L ? (not_head A sig n))))
 #tin #tout * #t1 * * #_ #Ht1 * #t2 * #Ht2 * #_ #Htout
 (* we start looking into Rmitl *)
 #ls #a #rs #Htin (* tin is a midtape *)
-#Hhead #Hreg #no_rightof #Hnohead_ls #Hnohead_rs 
-cut (regular_i sig n (a::ls) i)
+#Hheada #Hreg #no_rightof #Hnohead_ls #Hnohead_rs 
+cut (regular_i ? (S n) (a::ls) i)
   [cases (Hreg i) * // 
    cases (true_or_false (nth i ? (vec … a) (blank ?) == (blank ?))) #Htest
     [#_ @daemon (* absurd, since hd rs non e' blank *)
@@ -299,12 +334,10 @@ lapply (Htout … Ht2) -Htout -Ht2 *
   [(* the current character on trace i holds the head-mark.
       The case is absurd, since b0 is the head of rs2, that is a sublist of rs, 
       and the head-mark is not in rs *)
-   * #H3 @False_ind @(absurd (nth n ? (vec … b0) (blank sig) = head ?)) 
-     [@(\P ?) @injective_notb @H3 ]
-   @Hnohead_rs >H2 >trace_append @mem_append_l2 
+   * #H3 @False_ind @(absurd (true=false)) [2://] <H3 @sym_eq
+   <(notb_notb true) @(eq_f … notb) @Hnohead_rs >H2 >trace_append @mem_append_l2 
    lapply Hb0 cases rs2 
-    [whd in match (hd ???); #H >H in H3; whd in match (no_head ???); 
-     >all_blank_n normalize -H #H destruct (H); @False_ind
+    [>hd_nil #H >H in H3; >not_head_all_blanks #Habs destruct (Habs)
     |#c #r #H4 %1 >H4 //
     ]
   |* 
@@ -312,43 +345,43 @@ lapply (Htout … Ht2) -Htout -Ht2 *
    (* cut (trace sig n j (a1::ls20)=trace sig n j (ls1@b::ls2)) *)
    * #ls10 * #a1 * #ls20 * * * #Hls20 #Ha1 #Hnh #Htout
    cut (∀j.j ≠ i →
-      trace sig n j (reverse (multi_sig sig n) rs1@b::ls2) = 
-      trace sig n j (ls10@a1::ls20))
+      trace ? (S n) j (reverse (multi_sig (TA A sig) (S n)) rs1@b::ls2) = 
+      trace ? (S n) j (ls10@a1::ls20))
     [#j #ineqj >append_cons <reverse_cons >trace_def <map_append <reverse_map
-     lapply (trace_shift_neq …lt_in ? (sym_not_eq … ineqj) … Hrss) [//] #Htr
+     lapply (trace_shift_neq … (le_S … lt_in) ? (sym_not_eq … ineqj) … Hrss) [//] #Htr
      <(trace_def …  (b::rs1)) <Htr >reverse_map >map_append @eq_f @Hls20 ] 
    #Htracej
-   cut (trace sig n i (reverse (multi_sig sig n) (rs1@[b0])@ls2) = 
-        trace sig n i (ls10@a1::ls20))
+   cut (trace ? (S n) i (reverse (multi_sig (TA A sig) (S n)) (rs1@[b0])@ls2) = 
+        trace ? (S n) i (ls10@a1::ls20))
     [>trace_def <map_append <reverse_map <map_append <(trace_def … [b0]) 
-     cut (trace sig n i [b0] = [blank ?]) [@daemon] #Hcut >Hcut
-     lapply (trace_shift … lt_in … Hrss) [//] whd in match (tail ??); #Htr <Htr
+     cut (trace ? (S n) i [b0] = [blank ?]) [@daemon] #Hcut >Hcut
+     lapply (trace_shift … (le_S … lt_in) … Hrss) [//] whd in match (tail ??); #Htr <Htr
      >reverse_map >map_append <trace_def <Hls20 % 
     ] 
    #Htracei
    cut (∀j. j ≠ i →
-      (trace sig n j (reverse (multi_sig sig n) rs11) = trace sig n j ls10) ∧ 
-      (trace sig n j (ls1@b::ls2) = trace sig n j (a1::ls20)))
+      (trace ? (S n) j (reverse (MTA A sig (S n)) rs11) = trace ? (S n) j ls10) ∧ 
+      (trace ? (S n) j (ls1@b::ls2) = trace ? (S n) j (a1::ls20)))
    [@daemon (* si fa 
      #j #ineqj @(first_P_to_eq ? (λx. x ≠ head ?))
       [lapply (Htracej … ineqj) >trace_def in ⊢ (%→?); <map_append 
        >trace_def in ⊢ (%→?); <map_append #H @H  
       | *) ] #H2
-  cut ((trace sig n i (b0::reverse ? rs11) = trace sig n i (ls10@[a1])) ∧ 
-      (trace sig n i (ls1@ls2) = trace sig n i ls20))
+  cut ((trace ? (S n) i (b0::reverse ? rs11) = trace ? (S n) i (ls10@[a1])) ∧ 
+      (trace ? (S n) i (ls1@ls2) = trace ? (S n) i ls20))
    [>H1 in Htracei; >reverse_append >reverse_single >reverse_append 
      >reverse_reverse >associative_append >associative_append
      @daemon
     ] #H3    
   cut (∀j. j ≠ i → 
-    trace sig n j (reverse (multi_sig sig n) ls10@rs2) = trace sig n j rs)
-    [#j #jneqi @(injective_append_l … (trace sig n j (reverse ? ls1)))
+    trace ? (S n) j (reverse ? ls10@rs2) = trace ? (S n) j rs)
+    [#j #jneqi @(injective_append_l … (trace ? (S n) j (reverse ? ls1)))
      >map_append >map_append >Hrs1 >H1 >associative_append 
      <map_append <map_append in ⊢ (???%); @eq_f 
      <map_append <map_append @eq_f2 // @sym_eq 
      <(reverse_reverse … rs11) <reverse_map <reverse_map in ⊢ (???%);
      @eq_f @(proj1 … (H2 j jneqi))] #Hrs_j
-   %{ls20} %{a1} %{(reverse ? (b0::ls10)@tail (multi_sig sig n) rs2)}
+   %{ls20} %{a1} %{(reverse ? (b0::ls10)@tail ? rs2)}
    %[%[%[%[%[@Htout
     |#j cases (decidable_eq_nat j i)
       [#eqji >eqji (* by cases wether a1 is blank *)
@@ -361,17 +394,17 @@ lapply (Htout … Ht2) -Htout -Ht2 *
         |@sym_eq @Hrs_j //
         ]
       ]]
-    |#j #lejn #jneqi <(Hls1 … lejn
+    |#j #lejn #jneqi <(Hls1 … (le_S_S … lejn)
      >to_blank_i_def >to_blank_i_def @eq_f @sym_eq @(proj2 … (H2 j jneqi))]
     |#j #lejn #jneqi >reverse_cons >associative_append >Hb0
      <to_blank_hd_cons >to_blank_i_def >to_blank_i_def @eq_f @Hrs_j //]
-    |<(Hls1 i) [2:@lt_to_le //] 
+    |<(Hls1 i) [2:@le_S //] 
      lapply (all_blank_after_blank … reg_ls1_i) 
        [@(\P ?) @daemon] #allb_ls2
      whd in match (to_blank_i ????); <(proj2 … H3)
      @daemon ]
     |>reverse_cons >associative_append  
-     cut (to_blank_i sig n i rs = to_blank_i sig n i (rs11@[b0])) [@daemon] 
+     cut (to_blank_i ? (S n) i rs = to_blank_i ? (S n) i (rs11@[b0])) [@daemon] 
      #Hcut >Hcut >(to_blank_i_chop  … b0 (a1::reverse …ls10)) [2: @Hb0blank]
      >to_blank_i_def >to_blank_i_def @eq_f 
      >trace_def >trace_def @injective_reverse >reverse_map >reverse_cons
@@ -380,14 +413,14 @@ lapply (Htout … Ht2) -Htout -Ht2 *
     ]
   |(*we do not find the head: this is absurd *)
    * #b1 * #lss * * #H2 @False_ind 
-   cut (∀x0. mem ? x0 (trace sig n n (b0::reverse ? rss@ls2)) → x0 ≠ head ?)
+   cut (∀x0. mem ? x0 (trace ? (S n) n (b0::reverse ? rss@ls2)) → is_head … x0 = false)
      [@daemon] -H2 #H2
-   lapply (trace_shift_neq sig n i n … lt_in … Hrss)
+   lapply (trace_shift_neq ? (S n) i n … (le_S … lt_in) … Hrss)
      [@lt_to_not_eq @lt_in | // ] 
    #H3 @(absurd 
-        (nth n ? (vec … (hd ? (ls1@[b]) (all_blank sig n))) (blank ?) = head ?))
+        (is_head  … (nth n ? (vec … (hd ? (ls1@[b]) (all_blanks … (S n)))) (blank ?)) = true))
      [>Hhead //
-     |@H2 >trace_def %2 <map_append @mem_append_l1 <reverse_map <trace_def 
+     |@eqnot_to_noteq @H2 >trace_def %2 <map_append @mem_append_l1 <reverse_map <trace_def 
       >H3 >H1 >trace_def >reverse_map >reverse_cons >reverse_append 
       >reverse_reverse >associative_append <map_append @mem_append_l2
       cases ls1 [%1 % |#x #ll %1 %]