Skip to content

Commit

Permalink
disable example_open_terms.v (broken on master)
Browse files Browse the repository at this point in the history
  • Loading branch information
gares authored Dec 1, 2024
1 parent 9779044 commit a48378d
Showing 1 changed file with 2 additions and 2 deletions.
4 changes: 2 additions & 2 deletions examples/example_open_terms.v
Original file line number Diff line number Diff line change
Expand Up @@ -219,7 +219,7 @@ Tactic Notation (at level 0) "repl" uconstr(x) "with" uconstr(y) :=

Tactic Notation (at level 0) "repl" uconstr(x) "with" uconstr(y) "by" tactic(t) :=
elpi replace ltac_open_term:(x) ltac_open_term:(y); try (simpl; t).

(*
Lemma hard_example : forall l, map (fun x => x + 1) l = map (fun x => 1 + x) l.
Proof.
intros l.
Expand All @@ -233,6 +233,6 @@ Proof.
repl (x + 0 + y) with (y + x) by ring.
reflexivity.
Qed.

*)
(* An extended version of this tactic by Y. Bertot can be found in the tests/
directory under the name test_open_terms.v *)

0 comments on commit a48378d

Please sign in to comment.