aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--tactics/coretactics.ml44
-rw-r--r--tactics/tactics.ml4
-rw-r--r--tactics/tactics.mli1
3 files changed, 9 insertions, 0 deletions
diff --git a/tactics/coretactics.ml4 b/tactics/coretactics.ml4
index e909a14c9..92d4960a7 100644
--- a/tactics/coretactics.ml4
+++ b/tactics/coretactics.ml4
@@ -42,6 +42,10 @@ TACTIC EXTEND vm_cast_no_check
[ "vm_cast_no_check" constr(c) ] -> [ Proofview.V82.tactic (Tactics.vm_cast_no_check c) ]
END
+TACTIC EXTEND native_cast_no_check
+ [ "native_cast_no_check" constr(c) ] -> [ Proofview.V82.tactic (Tactics.native_cast_no_check c) ]
+END
+
TACTIC EXTEND casetype
[ "casetype" constr(c) ] -> [ Tactics.case_type c ]
END
diff --git a/tactics/tactics.ml b/tactics/tactics.ml
index 536a10eaa..131730ebc 100644
--- a/tactics/tactics.ml
+++ b/tactics/tactics.ml
@@ -1731,6 +1731,10 @@ let vm_cast_no_check c gl =
let concl = pf_concl gl in
refine_no_check (Term.mkCast(c,Term.VMcast,concl)) gl
+let native_cast_no_check c gl =
+ let concl = pf_concl gl in
+ refine_no_check (Term.mkCast(c,Term.NATIVEcast,concl)) gl
+
let exact_proof c gl =
let c,ctx = Constrintern.interp_casted_constr (pf_env gl) (project gl) c (pf_concl gl)
diff --git a/tactics/tactics.mli b/tactics/tactics.mli
index b9a018418..896b33727 100644
--- a/tactics/tactics.mli
+++ b/tactics/tactics.mli
@@ -118,6 +118,7 @@ val intros_patterns : intro_patterns -> unit Proofview.tactic
val assumption : unit Proofview.tactic
val exact_no_check : constr -> tactic
val vm_cast_no_check : constr -> tactic
+val native_cast_no_check : constr -> tactic
val exact_check : constr -> unit Proofview.tactic
val exact_proof : Constrexpr.constr_expr -> tactic