aboutsummaryrefslogtreecommitdiffhomepage
path: root/plugins
diff options
context:
space:
mode:
Diffstat (limited to 'plugins')
-rw-r--r--plugins/cc/cctac.ml2
-rw-r--r--plugins/firstorder/ground.ml2
-rw-r--r--plugins/romega/const_omega.ml4
-rw-r--r--plugins/romega/const_omega.mli4
-rw-r--r--plugins/ssr/ssrcommon.ml2
5 files changed, 7 insertions, 7 deletions
diff --git a/plugins/cc/cctac.ml b/plugins/cc/cctac.ml
index 8642df684..7f8f60e46 100644
--- a/plugins/cc/cctac.ml
+++ b/plugins/cc/cctac.ml
@@ -187,7 +187,7 @@ let make_prb gls depth additionnal_terms =
let open Tacmach.New in
let env=pf_env gls in
let sigma=project gls in
- let state = empty depth {it = Proofview.Goal.goal (Proofview.Goal.assume gls); sigma } in
+ let state = empty depth {it = Proofview.Goal.goal gls; sigma } in
let pos_hyps = ref [] in
let neg_hyps =ref [] in
List.iter
diff --git a/plugins/firstorder/ground.ml b/plugins/firstorder/ground.ml
index d46201335..09147d606 100644
--- a/plugins/firstorder/ground.ml
+++ b/plugins/firstorder/ground.ml
@@ -37,7 +37,7 @@ let ground_tac solver startseq =
let () =
if Tacinterp.get_debug()=Tactic_debug.DebugOn 0
then
- let gl = { Evd.it = Proofview.Goal.goal (Proofview.Goal.assume gl); sigma = project gl } in
+ let gl = { Evd.it = Proofview.Goal.goal gl; sigma = project gl } in
Feedback.msg_debug (Printer.pr_goal gl)
in
tclORELSE (axiom_tac seq.gl seq)
diff --git a/plugins/romega/const_omega.ml b/plugins/romega/const_omega.ml
index 0d491d92b..0f5417e7d 100644
--- a/plugins/romega/const_omega.ml
+++ b/plugins/romega/const_omega.ml
@@ -223,7 +223,7 @@ let mk_N = function
module type Int = sig
val typ : constr Lazy.t
- val is_int_typ : [ `NF ] Proofview.Goal.t -> constr -> bool
+ val is_int_typ : Proofview.Goal.t -> constr -> bool
val plus : constr Lazy.t
val mult : constr Lazy.t
val opp : constr Lazy.t
@@ -231,7 +231,7 @@ module type Int = sig
val mk : Bigint.bigint -> constr
val parse_term : constr -> parse_term
- val parse_rel : [ `NF ] Proofview.Goal.t -> constr -> parse_rel
+ val parse_rel : Proofview.Goal.t -> constr -> parse_rel
(* check whether t is built only with numbers and + * - *)
val get_scalar : constr -> Bigint.bigint option
end
diff --git a/plugins/romega/const_omega.mli b/plugins/romega/const_omega.mli
index 5ba063d9d..ecddc55de 100644
--- a/plugins/romega/const_omega.mli
+++ b/plugins/romega/const_omega.mli
@@ -105,7 +105,7 @@ module type Int =
(* the coq type of the numbers *)
val typ : constr Lazy.t
(* Is a constr expands to the type of these numbers *)
- val is_int_typ : [ `NF ] Proofview.Goal.t -> constr -> bool
+ val is_int_typ : Proofview.Goal.t -> constr -> bool
(* the operations on the numbers *)
val plus : constr Lazy.t
val mult : constr Lazy.t
@@ -116,7 +116,7 @@ module type Int =
(* parsing a term (one level, except if a number is found) *)
val parse_term : constr -> parse_term
(* parsing a relation expression, including = < <= >= > *)
- val parse_rel : [ `NF ] Proofview.Goal.t -> constr -> parse_rel
+ val parse_rel : Proofview.Goal.t -> constr -> parse_rel
(* Is a particular term only made of numbers and + * - ? *)
val get_scalar : constr -> Bigint.bigint option
end
diff --git a/plugins/ssr/ssrcommon.ml b/plugins/ssr/ssrcommon.ml
index d25ecee06..9822da1c7 100644
--- a/plugins/ssr/ssrcommon.ml
+++ b/plugins/ssr/ssrcommon.ml
@@ -1061,7 +1061,7 @@ let () = CLexer.set_keyword_state frozen_lexer ;;
(** Basic tactics *)
let rec fst_prod red tac = Proofview.Goal.nf_enter begin fun gl ->
- let concl = Proofview.Goal.concl (Proofview.Goal.assume gl) in
+ let concl = Proofview.Goal.concl gl in
match EConstr.kind (Proofview.Goal.sigma gl) concl with
| Prod (id,_,tgt) | LetIn(id,_,_,tgt) -> tac id
| _ -> if red then Tacticals.New.tclZEROMSG (str"No product even after head-reduction.")