Commit 95f083a 1 parent 44efa82 commit 95f083a Copy full SHA for 95f083a
File tree 3 files changed +5
-8
lines changed
3 files changed +5
-8
lines changed Original file line number Diff line number Diff line change @@ -45,10 +45,6 @@ Definition eqmodp (x y : int) := modp x = modp y.
45
45
Definition eq_Zmodp (x y : Zmodp) := (x = y).
46
46
Arguments eq_Zmodp /.
47
47
48
- (* Axiom (eqp_refl : Reflexive eqmodp). *)
49
- (* Axiom (eqp_sym : Symmetric eqmodp). *)
50
- (* Axiom (eqp_trans : Transitive eqmodp). *)
51
-
52
48
Notation "0" := zero : int_scope.
53
49
Notation "0" := zerop : Zmodp_scope.
54
50
Notation "x == y" := (eqmodp x%int y%int)
Original file line number Diff line number Diff line change @@ -23,14 +23,15 @@ Variables (to_nat : I -> nat) (of_nat : nat -> I).
23
23
24
24
Hypothesis to_natK : forall x, of_nat (to_nat x) = x.
25
25
Hypothesis of_nat0 : of_nat O = I0.
26
- Hypothesis of_natS : forall x n, of_nat n = x -> of_nat (S n) = IS x .
26
+ Hypothesis of_natS : forall n, of_nat (S n) = IS (of_nat n) .
27
27
28
- (* We only need/ (2a,3) which is morally that Nmap is a split injection *)
28
+ (* We only need (2a,3), so it suffices that to_nat is a retraction *)
29
29
Definition RI : Param2a3.Rel I nat :=
30
30
SplitSurj.toParamSym (SplitSurj.Build to_natK).
31
31
32
32
Definition RI0 : RI I0 O. Proof . exact of_nat0. Qed .
33
- Definition RIS m n : RI m n -> RI (IS m) (S n). Proof . exact: of_natS. Qed .
33
+ Definition RIS m n : RI m n -> RI (IS m) (S n).
34
+ Proof . by move=> <-; apply: of_natS. Qed .
34
35
35
36
Trocq Use RI RI0 RIS.
36
37
Original file line number Diff line number Diff line change @@ -19,7 +19,7 @@ From Trocq_examples Require Import N.
19
19
Set Universe Polymorphism.
20
20
21
21
(* the best we can do to link these types is (4,4), but
22
- we only need (2a,3) which is morally that Nmap is a split injection *)
22
+ we only need (2a,3) si ut suffices that N.to_nat is a retraction *)
23
23
Definition RN : Param2a3.Rel N nat :=
24
24
SplitSurj.toParamSym (SplitSurj.Build N.to_natK).
25
25
You can’t perform that action at this time.
0 commit comments