-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathPolTac.v
71 lines (56 loc) · 1.42 KB
/
PolTac.v
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
27
28
29
30
31
32
33
34
35
36
37
38
39
40
41
42
43
44
45
46
47
48
49
50
51
52
53
54
55
56
57
58
59
60
61
62
63
64
65
66
67
68
69
70
71
Require Export ArithRing.
Require Export NArithRing.
Require Import NatSignTac.
Require Import NSignTac.
Require Import ZSignTac.
Require Import RSignTac.
Ltac sign_tac :=
nsign_tac
|| Nsign_tac
|| zsign_tac
|| rsign_tac.
Ltac hyp_sign_tac H :=
hyp_nsign_tac H
|| hyp_Nsign_tac H
|| hyp_zsign_tac H
|| hyp_rsign_tac H.
Require Import NatPolS.
Require Import NPolS.
Require Import ZPolS.
Require Import RPolS.
Ltac pols := npols || Npols || zpols || rpols.
Ltac hyp_pols H :=
hyp_npols H
|| hyp_Npols H
|| hyp_zpols H
|| hyp_rpols H.
Require Import NatPolF.
Require Import NPolF.
Require Import ZPolF.
Require Import RPolF.
Ltac polf := npolf || Npolf || zpolf || rpolf.
Ltac hyp_polf H :=
hyp_npolf H
|| hyp_Npolf H
|| hyp_zpolf H
|| hyp_rpolf H.
Require Import NatPolR.
Require Import NPolR.
Require Import ZPolR.
Require Import RPolR.
Ltac polr term :=
match goal with
| [ |- ?G ] =>
let u := npol_is_compare G in npolr term
|| let u := Npol_is_compare G in Npolr term
|| let u := zpol_is_compare G in zpolr term
|| let u := rpol_is_compare G in rpolr term
end.
Ltac polrx term dir1 dir2 occ :=
match goal with
| [ |- ?G ] =>
let u := npol_is_compare G in npolrx term dir1 dir2 occ
|| let u := Npol_is_compare G in Npolrx term dir1 dir2 occ
|| let u := zpol_is_compare G in zpolrx term dir1 dir2 occ
|| let u := rpol_is_compare G in rpolrx term dir1 dir2 occ
end.