diff options
| author | Matthieu Sozeau | 2014-06-23 13:01:31 +0200 |
|---|---|---|
| committer | Matthieu Sozeau | 2014-06-23 13:10:02 +0200 |
| commit | db37c9f3f32ae7a2abcd5e1a3f6239eddb5e1768 (patch) | |
| tree | 6eaead7c3cd3b61ec54295a9037a4ef568b5dedb /plugins/btauto | |
| parent | 0b1507b16da38e883d63802db7c013e2c09665fd (diff) | |
Fix semantics of change p with c to typecheck c at each specific occurrence of p,
avoiding unwanted universe constraints in presence of universe polymorphic constants.
Fixing HoTT bugs # 36, 54 and 113.
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 6a0f4d8526..dbd89019e2 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_in_concl None changed_gl); + Proofview.V82.tactic (Tactics.change_concl changed_gl); Proofview.V82.tactic (Tactics.apply (Lazy.force soundness)); Proofview.V82.tactic (Tactics.normalise_vm_in_concl); try_unification env |
