aboutsummaryrefslogtreecommitdiff
path: root/src/Util/ZUtil/Tactics/PrimeBound.v
blob: f914ed7c838aaa9aad10bf69828e05e1b63d8113 (plain)
1
2
3
4
5
6
7
Require Import Coq.omega.Omega Coq.ZArith.Znumtheory.

Module Z.
  Ltac prime_bound := match goal with
  | [ H : prime ?p |- _ ] => pose proof (prime_ge_2 p H); try omega
  end.
End Z.