]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/formal_topology/overlap/basic_topologies.ma
eq over SET1 and SET no longer used
[helm.git] / helm / software / matita / contribs / formal_topology / overlap / basic_topologies.ma
index 26562cbb41805565c6eec931d6c7ad488ba3c325..4b53407d1f11e95c6b0deb713a597bef3ee653c9 100644 (file)
@@ -34,7 +34,7 @@ record continuous_relation (S,T: basic_topology) : Type1 ≝
    reduced: ∀U. U = J ? U → image ?? cont_rel U = J ? (image ?? cont_rel U);
    saturated: ∀U. U = A ? U → minus_star_image ?? cont_rel U = A ? (minus_star_image ?? cont_rel U)
  }. 
-
+(*
 definition continuous_relation_setoid: basic_topology → basic_topology → setoid1.
  intros (S T); constructor 1;
   [ apply (continuous_relation S T)
@@ -202,4 +202,5 @@ theorem continuous_relation_eqS:
   [2,4: intros; apply saturation_monotone; try (apply A_is_saturation); apply Hcut;]
  apply Hcut2; assumption.
 qed.
+*)
 *)
\ No newline at end of file