]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/library/formal_topology/o-algebra.ma
update in groud_2 and models
[helm.git] / helm / software / matita / library / formal_topology / o-algebra.ma
index 67ff5140e1f12fddc135b00a193b5a817913086c..fb508aa92b23c61b90dc280ab72297416ca177d9 100644 (file)
@@ -241,21 +241,12 @@ intros; apply (or_f ?? c);
 qed.
 coercion arrows1_of_ORelation_setoid.
 
-notation "r \sup *" non associative with precedence 90 for @{'OR_f_star $r}.
-notation > "r *" non associative with precedence 90 for @{'OR_f_star $r}.
-
-notation "r \sup (⎻* )" non associative with precedence 90 for @{'OR_f_minus_star $r}.
-notation > "r⎻*" non associative with precedence 90 for @{'OR_f_minus_star $r}.
-
-notation "r \sup ⎻" non associative with precedence 90 for @{'OR_f_minus $r}.
-notation > "r⎻" non associative with precedence 90 for @{'OR_f_minus $r}.
-
 interpretation "o-relation f⎻*" 'OR_f_minus_star r = (fun12 ?? (or_f_minus_star ? ?) r).
 interpretation "o-relation f⎻" 'OR_f_minus r = (fun12 ?? (or_f_minus ? ?) r).
 interpretation "o-relation f*" 'OR_f_star r = (fun12 ?? (or_f_star ? ?) r).
 
 definition or_prop1 : ∀P,Q:OAlgebra.∀F:ORelation_setoid P Q.∀p,q.
-   (F p ≤ q) = (p ≤ F* q).
+   (F p ≤ q) =_1 (p ≤ F* q).
 intros; apply (or_prop1_ ?? F p q);
 qed.