]> matita.cs.unibo.it Git - helm.git/blobdiff - matita/matita/lib/formal_topology/basic_topologies_to_o-basic_topologies.ma
update in ground_2
[helm.git] / matita / matita / lib / formal_topology / basic_topologies_to_o-basic_topologies.ma
index 0aeb58c737a459c5b691a21561a37ba199cfa610..6b07dfeb0863a9c493d9b71d90bb42361054de7d 100644 (file)
@@ -15,7 +15,7 @@
 include "formal_topology/basic_topologies.ma".
 include "formal_topology/o-basic_topologies.ma".
 include "formal_topology/relations_to_o-algebra.ma".
-
+(*
 definition o_basic_topology_of_basic_topology: basic_topology → Obasic_topology.
  intros (b); constructor 1;
   [ apply (POW' b) | apply (A b) | apply (J b);
@@ -29,7 +29,7 @@ definition o_continuous_relation_of_continuous_relation:
   [ apply (orelation_of_relation ?? c) | apply (reduced ?? c) | apply (saturated ?? c) ]
 qed.
 
-axiom daemon: ⊥. (*FG: alla faccia del costruttivismo *)
+axiom daemon: False.
 
 lemma o_continuous_relation_of_continuous_relation_morphism :
   ∀S,T:category2_of_category1 BTop.
@@ -89,3 +89,4 @@ theorem BTop_to_OBTop_full: full2 ?? BTop_to_OBTop.
    unfold image_coercion; cases Hg; whd; simplify; intro; simplify;
 qed.
 *)
+