X-Git-Url: http://matita.cs.unibo.it/gitweb/?a=blobdiff_plain;f=helm%2Fsoftware%2Fmatita%2Flibrary%2Fdecidable_kit%2Feqtype.ma;h=6aa3ff59fd2bf57600a558665606f7aa20e8b626;hb=e78cf74f8976cf0ca554f64baa9979d0423ee927;hp=4b248a97e13799b02387f6297f1d5c06483af710;hpb=9eabe046c1182960de8cfdba96c5414224e3a61e;p=helm.git diff --git a/helm/software/matita/library/decidable_kit/eqtype.ma b/helm/software/matita/library/decidable_kit/eqtype.ma index 4b248a97e..6aa3ff59f 100644 --- a/helm/software/matita/library/decidable_kit/eqtype.ma +++ b/helm/software/matita/library/decidable_kit/eqtype.ma @@ -50,7 +50,7 @@ definition nat_eqType : eqType ≝ mk_eqType ? ? eqbP. (* XXX le coercion nel cast non vengono inserite *) definition nat_canonical_eqType : nat → nat_eqType := λn : nat.(n : sort nat_eqType). -coercion cic:/matita/decidable_kit/eqtype/nat_canonical_eqType.con. +coercion nat_canonical_eqType. definition bcmp ≝ λx,y:bool. match x with [ true ⇒ y | false => notb y ]. @@ -68,7 +68,7 @@ qed. definition bool_eqType : eqType ≝ mk_eqType ? ? bcmpP. definition bool_canonical_eqType : bool → bool_eqType := λb : bool.(b : sort bool_eqType). -coercion cic:/matita/decidable_kit/eqtype/bool_canonical_eqType.con. +coercion bool_canonical_eqType. (* ### subtype of an eqType ### *) @@ -81,8 +81,7 @@ notation "{x, h}" right associative with precedence 80 for @{'sig $x $h}. -interpretation "sub_eqType" 'sig x h = - (cic:/matita/decidable_kit/eqtype/sigma.ind#xpointer(1/1/1) _ _ x h). +interpretation "sub_eqType" 'sig x h = (mk_sigma ? ? x h). (* restricting an eqType gives an eqType *) lemma sigma_eq_dec : ∀d:eqType.∀p.∀x,y:sigma d p. @@ -136,7 +135,7 @@ qed. definition option_eqType : eqType → eqType ≝ λd:eqType.mk_eqType ? ? (ocmpP d). definition option_canonical_eqType : ∀d:eqType.d → option_eqType d ≝ λd:eqType.λx:d.(Some ? x : sort (option_eqType d)). -coercion cic:/matita/decidable_kit/eqtype/option_canonical_eqType.con. +coercion option_canonical_eqType. (* belle le coercions! *) definition test_canonical_option_eqType ≝