1 2 3 4 5 6 7 8 9 10 11 12 13 14 15 16 17 18 19 20 21 22 23 24 25 26
|
Require Import Ltac2.Ltac2.
(** Test for quotations *)
Ltac2 ref0 () := reference:(&x).
Ltac2 ref1 () := reference:(nat).
Ltac2 ref2 () := reference:(Datatypes.nat).
Fail Ltac2 ref () := reference:(i_certainly_dont_exist).
Fail Ltac2 ref () := reference:(And.Me.neither).
Goal True.
Proof.
let x := constr:(I) in
let y := constr:((fun z => z) $x) in
Control.refine (fun _ => y).
Qed.
Goal True.
Proof.
(** Here, Ltac2 should not put its variables in the same environment as
Ltac1 otherwise the second binding fails as x is bound but not an
ident. *)
let x := constr:(I) in
let y := constr:((fun x => x) $x) in
Control.refine (fun _ => y).
Qed.
|