diff options
author | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-12-07 18:32:56 +0100 |
---|---|---|
committer | Hugo Herbelin <Hugo.Herbelin@inria.fr> | 2014-12-07 18:39:31 +0100 |
commit | 2fa05a8d300f5c0d375a558a8bced972eea4bfaf (patch) | |
tree | ecc7fa89b5f4be1bcc045fcd0d75e2b20f289566 /plugins/btauto | |
parent | 2acc6327e4d8a05898b75cb3abb47b7941ec420a (diff) |
Moving change_in_concl, change_in_hyp, change_concl to Proofview.tactic.
Diffstat (limited to 'plugins/btauto')
-rw-r--r-- | plugins/btauto/refl_btauto.ml | 2 |
1 files changed, 1 insertions, 1 deletions
diff --git a/plugins/btauto/refl_btauto.ml b/plugins/btauto/refl_btauto.ml index 6abf96dce..57268a9cf 100644 --- a/plugins/btauto/refl_btauto.ml +++ b/plugins/btauto/refl_btauto.ml @@ -247,7 +247,7 @@ module Btauto = struct let fr = reify env fr in let changed_gl = Term.mkApp (c, [|typ; fl; fr|]) in Tacticals.New.tclTHENLIST [ - Proofview.V82.tactic (Tactics.change_concl changed_gl); + Tactics.change_concl changed_gl; Tactics.apply (Lazy.force soundness); Proofview.V82.tactic (Tactics.normalise_vm_in_concl); try_unification env |