]> matita.cs.unibo.it Git - helm.git/blobdiff - helm/software/matita/nlibrary/sets/sets.ma
fixed coercion mechanism w.r.t. undo/require
[helm.git] / helm / software / matita / nlibrary / sets / sets.ma
index f3bd3b8898e35dd52f4f3d175ff79caf9690ca25..f140ef7700b7ca3b426debca3612628d8ac7f876 100644 (file)
@@ -39,7 +39,6 @@ ndefinition big_union ≝ λA,B.λT:Ω^A.λf:A → Ω^B.{ x | ∃i. i ∈ T ∧
 ndefinition big_intersection ≝ λA,B.λT:Ω^A.λf:A → Ω^B.{ x | ∀i. i ∈ T → x ∈ f i }.
 
 ndefinition full_set: ∀A. Ω^A ≝ λA.{ x | True }.
-ncoercion full_set : ∀A:Type[0]. Ω^A ≝ full_set on A: Type[0] to (Ω^?).
 
 nlemma subseteq_refl: ∀A.∀S: Ω^A. S ⊆ S.
  #A; #S; #x; #H; nassumption.
@@ -62,6 +61,9 @@ nqed.
 
 include "sets/setoids1.ma".
 
+(* this has to be declared here, so that it is combined with carr *)
+ncoercion full_set : ∀A:Type[0]. Ω^A ≝ full_set on A: Type[0] to (Ω^?).
+
 ndefinition powerclass_setoid: Type[0] → setoid1.
  #A; @[ napply (Ω^A)| napply seteq ]
 nqed.