]> matita.cs.unibo.it Git - helm.git/commitdiff
- notation fixed according to the new stricter semantics
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Thu, 19 Jun 2008 16:32:36 +0000 (16:32 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Thu, 19 Jun 2008 16:32:36 +0000 (16:32 +0000)
- generalize no longer required before case

helm/software/matita/contribs/dama/dama/cprop_connectives.ma
helm/software/matita/contribs/dama/dama/models/nat_dedekind_sigma_complete.ma
helm/software/matita/contribs/dama/dama/models/nat_lebesgue.ma
helm/software/matita/contribs/dama/dama/ordered_uniform.ma
helm/software/matita/contribs/dama/dama/property_sigma.ma
helm/software/matita/contribs/dama/dama/sequence.ma
helm/software/matita/contribs/dama/dama/uniform.ma

index 9e0e4b5fbb8e19c245c707d29f931923e91f2579..aabf6e79e08906331e8883e659a79f6c5ac19f6c 100644 (file)
@@ -28,14 +28,14 @@ interpretation "constructive and" 'and x y = (And x y).
 inductive And3 (A,B,C:CProp) : CProp ≝
  | Conj3 : A → B → C → And3 A B C.
 
-notation < "a ∧ b ∧ c" left associative with precedence 35 for @{'and3 $a $b $c}.
+notation < "a ∧ b ∧ c" with precedence 35 for @{'and3 $a $b $c}.
  
 interpretation "constructive ternary and" 'and3 x y z = (Conj3 x y z).
 
 inductive And4 (A,B,C,D:CProp) : CProp ≝
  | Conj4 : A → B → C → D → And4 A B C D.
 
-notation < "a ∧ b ∧ c ∧ d" left associative with precedence 35 for @{'and4 $a $b $c $d}.
+notation < "a ∧ b ∧ c ∧ d" with precedence 35 for @{'and4 $a $b $c $d}.
  
 interpretation "constructive quaternary and" 'and4 x y z t = (Conj4 x y z t).
 
index 04b861d41cea7e497feb7be6dfcfbc5f881a019d..0908b6f7079ae8f2acf97cfac5758717b3124054 100644 (file)
@@ -52,11 +52,8 @@ letin m ≝ (hide ? (
    ∀i:nat.∃j:nat.spec i j));unfold spec in aux ⊢ %;
 [1: apply (H2 pred nP);
 |4: unfold X in H2; clear H4 n aux spec H3 H1 H X;
-    generalize in match H2;
-    generalize in match Hs;
-    generalize in match a;
-    clear H2 Hs a; cases u; intros (a Hs H);
-    [1: left; split; [apply le_n] 
+    cases u in H2 Hs a ⊢ %; intros (a Hs H);
+    [1: left; split; [apply le_n]
         generalize in match H;
         generalize in match Hs;
         rewrite > (?:s = O); 
@@ -68,7 +65,7 @@ letin m ≝ (hide ? (
         apply (trans_le ??? (os_le_to_nat_le ?? H1));
         apply le_plus_n_r;] 
 |2,3: clear H6;
-    generalize in match H5; clear H5; cases (aux n1); intros;
+    cases (aux n1) in H5 ⊢ %; intros;
     change in match (a 〈w,H5〉) in H6 ⊢ % with (a w);
     cases H5; clear H5; cases H7; clear H7;
     [1: left; split; [ apply (le_S ?? H5); | assumption]
index 228392dda8a8c7254fc5c1abcd8d2d14fb595c4d..7e059c03d96d2bc37c86a73ae02d5189dd272e9e 100644 (file)
@@ -17,7 +17,7 @@ include "models/nat_order_continuous.ma".
 
 alias symbol "pair" = "dependent pair".
 theorem nat_lebesgue_oc:
-   ∀a:sequence ℕ.∀l,u:nat_ordered_uniform_space.∀H:∀i:nat.a i ∈ [l,u]. 
+   ∀a:sequence ℕ.∀l,u:.∀H:∀i:nat.a i ∈ [l,u]. 
      ∀x:ℕ.a order_converges x → 
       x ∈ [l,u] ∧ 
       ∀h:x ∈ [l,u].
index 8aacb5b59214bafbb89911b4ca3f9530823f06d8..326681b2608d2ce0c0bc673d41aa43d73cd8b04e 100644 (file)
@@ -96,7 +96,7 @@ lemma bs_of_ss:
  ∀O:ordered_set.∀u,v:O.{[u,v]} square → (bishop_set_of_ordered_set O) square ≝ 
   λO:ordered_set.λu,v:O.λb:{[u,v]} square.〈fst(fst b),fst(snd b)〉.
 
-notation < "x \sub \neq" left associative with precedence 91 for @{'bsss $x}.
+notation < "x \sub \neq" with precedence 91 for @{'bsss $x}.
 interpretation "bs_of_ss" 'bsss x = (bs_of_ss _ _ _ x).
 
 alias symbol "square" (instance 7) = "ordered set square".
@@ -108,7 +108,7 @@ lemma ss_of_bs:
  λO:ordered_set.λu,v:O.
   λb:(O:bishop_set) square.λH1,H2.〈〈fst b,H1〉,〈snd b,H2〉〉.
 
-notation < "x \sub \nleq" left associative with precedence 91 for @{'ssbs $x}.
+notation < "x \sub \nleq" with precedence 91 for @{'ssbs $x}.
 interpretation "ss_of_bs" 'ssbs x = (ss_of_bs _ _ _ x _ _).
 
 lemma segment_ordered_uniform_space: 
index ba90bb0ab50097e864bdf9c884902aa049098c44..67209928116df8aec54e7a70e5304a0011d257e1 100644 (file)
@@ -77,9 +77,8 @@ letin m ≝ (hide ? (let rec aux (i:nat) : nat ≝
       intros; lapply (H5 i j) as H14;
         [2: apply (max_le_l ??? H6);|3:apply (max_le_l ??? H7);]
       cases (le_to_or_lt_eq ?? H10); [2: destruct H11; destruct H4; assumption]
-      generalize in match H6; generalize in match H7;
-      cases (aux n1); simplify in ⊢ (? (? ? %) ?→? (? ? %) ?→?); intros;
-      apply H12; [3: apply le_S_S_to_le; assumption]
+      cases (aux n1) in H6 H7 ⊢ %; simplify in ⊢ (? (? ? %) ?→? (? ? %) ?→?); intros;
+      apply H6; [3: apply le_S_S_to_le; assumption]
       apply lt_to_le; apply (max_le_r w1); assumption;
   |4: intros; clear H6; rewrite > H4 in H5; 
       rewrite < (le_n_O_to_eq ? H11); apply H5; assumption;] 
index c643154810acf3dc5ad92c452632dea28187ba5c..39c40194bca3c8db2133e149a8aa2a206fb8b979 100644 (file)
@@ -22,16 +22,13 @@ definition fun_of_seq: ∀O:Type.sequence O → nat → O ≝
 
 coercion cic:/matita/dama/sequence/fun_of_seq.con 1.
 
-notation < "hvbox((\lfloor p \rfloor) \sub ident i)"
-  left associative with precedence 70
+notation < "hvbox((\lfloor p \rfloor) \sub ident i)" with precedence 70
 for @{ 'sequence (\lambda ${ident i} : $t . $p)}.
 
-notation > "hvbox((\lfloor p \rfloor) \sub ident i)"
-  left associative with precedence 70
+notation > "hvbox((\lfloor p \rfloor) \sub ident i)" with precedence 70
 for @{ 'sequence (\lambda ${ident i} . $p)}.
 
-notation > "hvbox(\lfloor ident i, p \rfloor)"
-  left associative with precedence 70
+notation > "hvbox(\lfloor ident i, p \rfloor)" with precedence 70
 for @{ 'sequence (\lambda ${ident i} . $p)}.
   
 notation "a \sub i" left associative with precedence 70 
index faba6d83a68be9cc9f2e45d04b4a661072961b2b..ed9e6fe5d1d60a66ddf205d8e1bbcbe7f0ffd113 100644 (file)
@@ -35,12 +35,10 @@ definition invert_bs_relation ≝
   λC:bishop_set.λU:C square → Prop.
     λx:C square. U 〈snd x,fst x〉.
     
-notation < "s \sup (-1)"  left associative with precedence 70
-  for @{ 'invert $s }.
-notation < "s \sup (-1) x"  left associative with precedence 70
+notation < "s \sup (-1)"  with precedence 70 for @{ 'invert $s }.
+notation < "s \sup (-1) x"  with precedence 70
   for @{ 'invert_appl $s $x}. 
-notation > "'inv'" right associative with precedence 70
-  for @{ 'invert_symbol  }.
+notation > "'inv'" with precedence 70 for @{ 'invert_symbol  }.
 interpretation "relation invertion" 'invert a = (invert_bs_relation _ a).
 interpretation "relation invertion" 'invert_symbol = (invert_bs_relation _).
 interpretation "relation invertion" 'invert_appl a x = (invert_bs_relation _ a x).