File: conv.v

package info (click to toggle)
coq 9.1.0%2Bdfsg-3
  • links: PTS, VCS
  • area: main
  • in suites: experimental
  • size: 35,964 kB
  • sloc: ml: 239,908; sh: 4,355; python: 2,985; ansic: 2,644; makefile: 874; lisp: 171; javascript: 63; xml: 24; sed: 2
file content (18 lines) | stat: -rw-r--r-- 617 bytes parent folder | download
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
Require Import Ltac2.Ltac2.

Definition foo : nat := 1.
Opaque foo.

Goal True /\ False.
  (* conversion works *)
  Control.assert_true (Unification.conv_full '4 '(2 + 2)).
  (* conversion fails *)
  Fail Control.assert_true (Unification.conv_full '4 '3).
  (* at most one goal must be focussed *)
  split. Fail all: Unification.conv_full '4 '(2 + 2).
  (* constants are respected *)
  Fail Control.assert_true (Unification.conv_current 'foo '1).
  Control.assert_true (Unification.conv_full 'foo '1).
  (* its the local env that is used *)
  pose (x := 1); Control.assert_true (Unification.conv_full '&x '1).
Abort.