]> matita.cs.unibo.it Git - helm.git/commitdiff
Dead code removed.
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Fri, 18 Apr 2008 18:31:58 +0000 (18:31 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Fri, 18 Apr 2008 18:31:58 +0000 (18:31 +0000)
helm/software/matita/contribs/POPLmark/Fsub/defn.ma

index 3bd8d2bdcdf75f2d83be67bd2077fc2b47c4948d..7907405ff9057c62e9644697ee0336eb10cb0764 100644 (file)
@@ -44,16 +44,6 @@ let rec subst_type_nat T U i \def
     | (Arrow T1 T2) \Rightarrow (Arrow (subst_type_nat T1 U i) (subst_type_nat T2 U i))
     | (Forall T1 T2) \Rightarrow (Forall (subst_type_nat T1 U i) (subst_type_nat T2 U (S i))) ].
 
-(*** height of T's syntactic tree ***)
-
-let rec t_len T \def
-  match T with
-     [(TVar n) \Rightarrow (S O)
-     |(TFree X) \Rightarrow (S O)
-     |Top \Rightarrow (S O)
-     |(Arrow T1 T2) \Rightarrow (S (max (t_len T1) (t_len T2)))
-     |(Forall T1 T2) \Rightarrow (S (max (t_len T1) (t_len T2)))].
-
 (*** definitions about lists ***)
 
 definition fv_env : (list bound) \to (list nat) \def
@@ -147,11 +137,6 @@ notation "hvbox(S [# n ↦ T])"
 interpretation "subst bound var" 'substvar S T n =
   (cic:/matita/Fsub/defn/subst_type_nat.con S T n).  
 
-notation "hvbox(|T|)"
-  non associative with precedence 30 for @{ 'tlen $T }.
-interpretation "type length" 'tlen T =
-  (cic:/matita/Fsub/defn/t_len.con T).  
-
 notation "hvbox(!X ⊴ T)"
   non associative with precedence 60 for @{ 'subtypebound $X $T }.
 interpretation "subtyping bound" 'subtypebound X T =
@@ -390,4 +375,4 @@ qed.
 
 lemma fv_append : ∀G,H.fv_env (G @ H) = (fv_env G @ fv_env H).
 intro;elim G;simplify;autobatch paramodulation;
-qed.
\ No newline at end of file
+qed.