]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/nlibrary/sets/sets.ma
...
[helm.git] / helm / software / matita / nlibrary / sets / sets.ma
index 623f676e96d944a4437dee92307063322e33c717..3d03887ec2e4a163292041486a977f596631b40c 100644 (file)
@@ -116,7 +116,8 @@ unification hint 0 ≔ A;
   (* ----------------------------------------------------- *) ⊢  
                  carr1 R ≡ ext_powerclass A.
 
-                
+interpretation "prop21 mem" 'prop2 l r = (prop21 (setoid1_of_setoid ?) (ext_powerclass_setoid ?) ? ? ???? l r).
+      
 (*
 ncoercion ext_carr' : ∀A.∀x:ext_powerclass_setoid A. Ω^A ≝ ext_carr 
 on _x : (carr1 (ext_powerclass_setoid ?)) to (Ω^?). 
@@ -159,7 +160,7 @@ unification hint 0 ≔ A,a,a'
 
 nlemma intersect_is_ext: ∀A. 𝛀^A → 𝛀^A → 𝛀^A.
  #A; #S; #S'; @ (S ∩ S');
- #a; #a'; #Ha; @; *; #H1; #H2; @
+ #a; #a'; #Ha; @; *; #H1; #H2; @ 
   [##1,2: napply (. Ha^-1‡#); nassumption;
 ##|##3,4: napply (. Ha‡#); nassumption]
 nqed.
@@ -192,8 +193,7 @@ unification hint 0 ≔
     fun21 (powerclass_setoid A) (powerclass_setoid A) (powerclass_setoid A) R B C 
   ≡ intersect ? B C.
 
-interpretation "prop21 mem" 'prop2 l r = (prop21 (setoid1_of_setoid ?) (ext_powerclass_setoid ?) ? ???? l r).
-interpretation "prop21 ext" 'prop2 l r = (prop21 (ext_powerclass_setoid ?) (ext_powerclass_setoid ?) ? ???? l r).
+interpretation "prop21 ext" 'prop2 l r = (prop21 (ext_powerclass_setoid ?) (ext_powerclass_setoid ?) ? ? ???? l r).
 
 nlemma intersect_is_ext_morph: 
  ∀A. binary_morphism1 (ext_powerclass_setoid A) (ext_powerclass_setoid A) (ext_powerclass_setoid A).
@@ -231,12 +231,13 @@ unification hint 0 ≔
           
 unification hint 0 ≔
   A, B : CPROP ⊢ iff A B ≡ eq_rel1 ? (eq1 CPROP) A B.    
-*)
     
 nlemma test: ∀U.∀A,B:𝛀^U. A ∩ B = A →
  ∀x,y. x=y → x ∈ A → y ∈ A ∩ B.
  #U; #A; #B; #H; #x; #y; #K; #K2;
-napply (. (prop21 ??? ? ???? K^-1 (H^-1‡#)));
+  alias symbol "prop2" = "prop21 mem".
+  alias symbol "invert" = "setoid1 symmetry".
+  napply (. K^-1‡H);
   nassumption;
 nqed. 
 
@@ -251,14 +252,16 @@ nlemma intersect_ok: ∀A. binary_morphism1 (ext_powerclass_setoid A) (ext_power
       ##|##3,4: napply (. Ha‡#); nassumption]##]
  ##| #a; #a'; #b; #b'; #Ha; #Hb; nwhd; @; #x; nwhd in ⊢ (% → %); #H
       [ alias symbol "invert" = "setoid1 symmetry".
-        napply (. ((#‡Ha^-1)‡(#‡Hb^-1))); nassumption
+        alias symbol "refl" = "refl".
+alias symbol "prop2" = "prop21".
+napply (. ((#‡Ha^-1)‡(#‡Hb^-1))); nassumption
       | napply (. ((#‡Ha)‡(#‡Hb))); nassumption ]##]
 nqed.
 
 (* unfold if intersect, exposing fun21 *)
 alias symbol "hint_decl" = "hint_decl_Type1".
 unification hint 0 ≔ 
-  A : setoid, B,C : qpowerclass A ⊢ 
+  A : setoid, B,C : ext_powerclass A ⊢ 
     pc A (fun21 …
             (mk_binary_morphism1 …
               (λS,S':qpowerclass_setoid A.mk_qpowerclass ? (S ∩ S') (mem_ok' ? (intersect_ok ? S S'))) 
@@ -271,7 +274,6 @@ nlemma test: ∀A:setoid. ∀U,V:qpowerclass A. ∀x,x':setoid1_of_setoid A. x=x
  #A; #U; #V; #x; #x'; #H; #p; napply (. (H^-1‡#)); nassumption.
 nqed.
 *)
-*)
 
 ndefinition image: ∀A,B. (carr A → carr B) → Ω^A → Ω^B ≝
  λA,B:setoid.λf:carr A → carr B.λSa:Ω^A.