]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/formal_topology/overlap/subsets.ma
1) Some reorganization.
[helm.git] / helm / software / matita / contribs / formal_topology / overlap / subsets.ma
index 41e29a4fb8ff756dd0ea0f00620d5a39b1fcd063..3aaf2d3d6b34b6da73f52a678e6cfb7d95c5f73b 100644 (file)
@@ -165,47 +165,3 @@ definition big_union:
      [ apply (. (#‡(e w))); apply x;
      | apply (. (#‡(e w)\sup -1)); apply x]]
 qed.
-
-(* incluso prima non funziona piu' nulla *)
-include "o-algebra.ma".
-
-definition SUBSETS: objs1 SET → OAlgebra.
- intro A; constructor 1;
-  [ apply (Ω \sup A);
-  | apply subseteq;
-  | apply overlaps;
-  | apply big_intersects;
-  | apply big_union;
-  | apply ({x | True});
-    simplify; intros; apply (refl1 ? (eq1 CPROP));
-  | apply ({x | False});
-    simplify; intros; apply (refl1 ? (eq1 CPROP));
-  | intros; whd; intros; assumption
-  | intros; whd; split; assumption
-  | intros; apply transitive_subseteq_operator; [2: apply f; | skip | assumption]
-  | intros; cases f; exists [apply w] assumption
-  | intros; intros 2; apply (f ? f1 i);
-  | intros; intros 2; apply f;
-    (* senza questa change, universe inconsistency *)
-    whd; change in ⊢ (? ? (λ_:%.?)) with (carr I);
-    exists; [apply i] assumption;
-  | intros 3; cases f;
-  | intros 3; constructor 1;
-  | intros; cases f; exists; [apply w]
-     [ assumption
-     | whd; intros; cases i; simplify; assumption]
-  | intros; split; intro;
-     [ cases f; cases x1;
-       (* senza questa change, universe inconsistency *)
-       change in ⊢ (? ? (λ_:%.?)) with (carr I);
-       exists [apply w1] exists [apply w] assumption;
-     | cases e; cases x; exists; [apply w1]
-        [ assumption
-        | (* senza questa change, universe inconsistency *)
-          whd; change in ⊢ (? ? (λ_:%.?)) with (carr I);
-          exists; [apply w] assumption]]
-  | intros; intros 2; cases (f (singleton ? a) ?);
-     [ exists; [apply a] [assumption | change with (a = a); apply refl1;]
-     | change in x1 with (a = w); change with (mem A a q); apply (. (x1 \sup -1‡#));
-       assumption]]
-qed.