Skip to content

Commit

Permalink
removing bug for now and silencing dev debug
Browse files Browse the repository at this point in the history
  • Loading branch information
CohenCyril committed Dec 10, 2023
1 parent 71f52d0 commit ed563c8
Show file tree
Hide file tree
Showing 3 changed files with 2 additions and 18 deletions.
Binary file modified artifact-clean.zip
Binary file not shown.
18 changes: 1 addition & 17 deletions examples/Vector_tuple.v
Original file line number Diff line number Diff line change
Expand Up @@ -258,16 +258,10 @@ Trocq Use Param_const.
Trocq Use Param01_paths.

Lemma head_const' : forall {n : nat} (z : Zp), head (const z (S n)) = z.
Proof. trocq. intro n. apply head_const. Qed.
Proof. trocq; exact: @head_const. Qed.

End HeadConst.



(* bug *)

Module bug.

Definition cons {A : Type} {n : nat} (a : A) (t : tuple A n) : tuple A (S n) := (t, a).

Definition Param_cons
Expand All @@ -292,16 +286,6 @@ Defined.
Trocq Use SR.
Trocq Use Param_cons.

Lemma append_comm_cons : forall {A : Type} {n1 n2 : nat}
(v1 : tuple A n1) (v2 : tuple A n2) (a : A),
@paths (tuple A (S (n1 + n2))) (cons a (append v1 v2)) (append (cons a v1) v2).
Proof.
Fail Timeout 1 trocq.
(* apply Vector.append_comm_cons. *)
Abort.

End bug.

(* bounded nat and bitvector *)
(* NB: we can use transitivity to make the proofs here too *)

Expand Down
2 changes: 1 addition & 1 deletion theories/Param.v
Original file line number Diff line number Diff line change
Expand Up @@ -155,7 +155,7 @@ Elpi Accumulate lp:{{
}}.

Elpi Accumulate lp:{{
solve InitialGoal NewGoals :- debug dbg.full => std.do! [
solve InitialGoal NewGoals :- debug dbg.none => std.do! [
InitialGoal = goal _Context _ G _ [],
util.when-debug dbg.full (coq.say "goal" G),
translate-goal G (pc map0 map1) G' GR,
Expand Down

0 comments on commit ed563c8

Please sign in to comment.