]> matita.cs.unibo.it Git - helm.git/commitdiff
1. new coercion(s) from CPropi to CProp
authorClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Fri, 16 Jan 2009 00:45:58 +0000 (00:45 +0000)
committerClaudio Sacerdoti Coen <claudio.sacerdoticoen@unibo.it>
Fri, 16 Jan 2009 00:45:58 +0000 (00:45 +0000)
2. fixed notation for subsetS
3. coercions still have problems: the coercion from objs1 REL is not
   accepted because it is identified with the coercion from objs1 SET

helm/software/matita/contribs/formal_topology/overlap/basic_pairs.ma
helm/software/matita/contribs/formal_topology/overlap/concrete_spaces.ma
helm/software/matita/contribs/formal_topology/overlap/cprop_connectives.ma

index a7be5cc6c5db889bf10e791e477f149e0095182c..6140e278ec5c30e0d8624d90c0b50624f67ccde9 100644 (file)
@@ -193,5 +193,5 @@ definition relS: ∀o: BP. binary_morphism1 (concr o) (Ω \sup (form o)) CPROP.
      | apply (. (#‡e1)‡(e‡#)); assumption]]
 qed.
 
-interpretation "basic pair relation for subsets" 'Vdash2 x y = (fun21 (concr _) __ (relS _) x y).
-interpretation "basic pair relation for subsets (non applied)" 'Vdash = (fun21 ___ (relS _)).
+interpretation "basic pair relation for subsets" 'Vdash2 x y c = (fun21 (concr _) __ (relS c) x y).
+interpretation "basic pair relation for subsets (non applied)" 'Vdash c = (fun21 ___ (relS c)).
index 07a067e73f5c62419d11a52eb529f4f9bd0b1af0..46e5378649a169845fdb74a3d79de5e14eda65d4 100644 (file)
 
 include "basic_pairs.ma".
 
-(* full_subset e' una coercion che non mette piu' *)
+(* carr1 e' necessario perche' ci sega via la coercion per gli oggetti di REL!
+   (confondendola con la coercion per gli oggetti di SET *)
 record concrete_space : Type1 ≝
  { bp:> BP;
-   converges: ∀a: concr bp.∀U,V: form bp. a ⊩ U → a ⊩ V → a ⊩ (U ↓ V);
-   all_covered: ∀x: concr bp. x ⊩ full_subset (form bp)
+   converges: ∀a: carr1 (concr bp).∀U,V: carr1 (form bp). a ⊩ U → a ⊩ V → a ⊩_bp (U ↓ V);
+   all_covered: ∀x: carr1 (concr bp). x ⊩ form bp
  }.
 
 record convergent_relation_pair (CS1,CS2: concrete_space) : Type1 ≝
index d6c7084b0f511eb92e293d97d80c747c5929a377..167c33317c8d4810e7cd0533e5b3aab7b0bf7b6f 100644 (file)
@@ -31,6 +31,12 @@ coercion Type_of_Type3.
 definition CProp0 : Type1 := Type0.
 definition CProp1 : Type2 := Type1.
 definition CProp2 : Type3 := Type2.
+definition CProp_of_CProp0: CProp0 → CProp ≝ λx.x.
+definition CProp_of_CProp1: CProp1 → CProp ≝ λx.x.
+definition CProp_of_CProp2: CProp2 → CProp ≝ λx.x.
+coercion CProp_of_CProp0.
+coercion CProp_of_CProp1.
+coercion CProp_of_CProp2.
 
 inductive Or (A,B:CProp0) : CProp0 ≝
  | Left : A → Or A B