]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/contribs/formal_topology/overlap/relations.ma
An hint moved to the right place.
[helm.git] / helm / software / matita / contribs / formal_topology / overlap / relations.ma
index eb60386fe3d1abc0831f7f747d7a5093062845c9..ed8b83bcbd1f3b17538cfe595ccf37d05f02efb0 100644 (file)
@@ -175,12 +175,6 @@ lemma extS_com: ∀o1,o2,o3,c1,c2,S. extS o1 o3 (c2 ∘ c1) S = extS o1 o2 c1 (e
 qed.
 *)
 
-lemma hint: ∀U. carr U → Type_OF_setoid1 ?(*(setoid1_of_SET U)*).
- [ apply setoid1_of_SET; apply U
- | intros; apply c;]
-qed.
-coercion hint.
-
 (* the same as ⋄ for a basic pair *)
 definition image: ∀U,V:REL. binary_morphism1 (arrows1 ? U V) (Ω \sup U) (Ω \sup V).
  intros; constructor 1;
@@ -327,4 +321,4 @@ definition orelation_of_relation: ∀o1,o2:REL. arrows1 ? o1 o2 → ORelation (S
      | cases x1; cases x2; clear x1 x2; exists; [apply w1]
         [ exists; [apply w] split; assumption;
         | assumption; ]]]
-qed. (*sistemare anche l'hint da un'altra parte *)
+qed.