Skip to content

Commit

Permalink
Better HB structure
Browse files Browse the repository at this point in the history
  • Loading branch information
thery committed Nov 2, 2023
1 parent 6035711 commit 6d3b322
Showing 1 changed file with 5 additions and 7 deletions.
12 changes: 5 additions & 7 deletions gauss_int.v
Original file line number Diff line number Diff line change
Expand Up @@ -223,6 +223,7 @@ We provide the subtype property.
*)

#[verbose]

Check warning on line 226 in gauss_int.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.1.0-coq-8.18)

Projection value has no head constant:

Check warning on line 226 in gauss_int.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.1.0-coq-8.18)

Ignoring canonical projection to vrefl_rect by isSub.SubK_subproof
HB.instance Definition _ := [isSub for algGI].

(**
Expand All @@ -244,12 +245,11 @@ canonical property for the predicate gaussInt
*)

HB.instance Definition _ := [Equality of GI by <:].
HB.instance Definition _ := [Choice of GI by <:].
HB.howto GI subComRingType.

HB.instance Definition _ := [Countable of GI by <:].

Check warning on line 250 in gauss_int.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.1.0-coq-8.18)

Ignoring canonical projection to inj_eqAxiom by hasDecEq.eqP in

Check warning on line 250 in gauss_int.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.1.0-coq-8.18)

Ignoring canonical projection to eq_op by hasDecEq.eq_op in

Check warning on line 250 in gauss_int.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.1.0-coq-8.18)

Ignoring canonical projection to isCountable.pickleK by

Check warning on line 250 in gauss_int.v

View workflow job for this annotation

GitHub Actions / build (mathcomp/mathcomp:2.1.0-coq-8.18)

Ignoring canonical projection to isCountable.unpickle by
HB.instance Definition _ := [SubChoice_isSubZmodule of GI by <:].
HB.instance Definition _ := [SubZmodule_isSubRing of GI by <:].
HB.instance Definition _ := [SubRing_isSubComRing of GI by <:].
HB.instance Definition _ := [SubChoice_isSubComRing of GI by <:].

(**
- Now we build the unitRing and comUnitRing structure of gauss
Expand Down Expand Up @@ -1259,8 +1259,6 @@ Coercion GI_of_ord i := let: OrdinalGI m _ := i in m.


HB.instance Definition _ := [isSub for GI_of_ord].
HB.instance Definition _ := [Equality of ordinalGI by <:].
HB.instance Definition _ := [Choice of ordinalGI by <:].
HB.instance Definition _ := [Countable of ordinalGI by <:].

Lemma ltn_ordGI (i : ordinalGI) : ('N i < n)%N.
Expand Down

0 comments on commit 6d3b322

Please sign in to comment.