Skip to content

Commit

Permalink
remove logs
Browse files Browse the repository at this point in the history
  • Loading branch information
adelaett committed Jan 22, 2024
1 parent 88e01d4 commit 83064ce
Showing 1 changed file with 9 additions and 5 deletions.
14 changes: 9 additions & 5 deletions theories/simulation_sred_to_cred.v
Original file line number Diff line number Diff line change
Expand Up @@ -1551,7 +1551,7 @@ Proof.
all: inversion Hs2; subst; eauto.
Qed.

Ltac info :=
(* Ltac info :=
match goal with
| [ |- plus cred ?s1 _ /\ _ ] =>
idtac s1 "//"
Expand All @@ -1560,7 +1560,9 @@ Ltac info :=
| [ |- cred ?s1 _ /\ _ ] =>
idtac s1 "//"
| _ => idtac
end.
end. *)

Ltac info := idtac.



Expand Down Expand Up @@ -1757,7 +1759,8 @@ Proof.

(* When no more progress is possible, we can finaly introduce the evar corresponding to the goal term. This is to avoid having variable completing our evar that escape the scope they were defined in. *)
| [ |- exists _, _] =>
idtac "---"; eexists
(* idtac "---"; *)
eexists
| _ =>
info;
solve [split; [eapply star_refl|];
Expand Down Expand Up @@ -2019,7 +2022,8 @@ Proof.

(* When no more progress is possible, we can finaly introduce the evar corresponding to the goal term. This is to avoid having variable completing our evar that escape the scope they were defined in. *)
| [ |- exists _, _] =>
let P := type of Hred_current in idtac "---"; idtac P "//"; eexists
(* let P := type of Hred_current in idtac "---"; idtac P "//"; *)
eexists
| _ =>
first[solve [split; [info; eapply star_refl|];
solve [
Expand All @@ -2038,7 +2042,7 @@ Proof.
end
(* For return cases *)
| econstructor; simpl; rewrite subst_env_cons; asimpl; eauto
]; idtac "ok"] | idtac "notok"]
](*; idtac "ok" *)] (* | idtac "notok" *)]
end.

all: try solve [ repeat match goal with
Expand Down

0 comments on commit 83064ce

Please sign in to comment.