aboutsummaryrefslogtreecommitdiffhomepage
diff options
context:
space:
mode:
-rw-r--r--plugins/cc/ccalgo.ml3
-rw-r--r--test-suite/bugs/closed/shouldsucceed/3054.v10
2 files changed, 12 insertions, 1 deletions
diff --git a/plugins/cc/ccalgo.ml b/plugins/cc/ccalgo.ml
index aba908d48..fbe31fe52 100644
--- a/plugins/cc/ccalgo.ml
+++ b/plugins/cc/ccalgo.ml
@@ -427,7 +427,8 @@ let rec add_term state t=
try Termhash.find uf.syms t with
Not_found ->
let b=next uf in
- let typ = pf_type_of state.gls (constr_of_term t) in
+ let trm = Termops.refresh_universes (constr_of_term t) in
+ let typ = pf_type_of state.gls trm in
let typ = canonize_name typ in
let new_node=
match t with
diff --git a/test-suite/bugs/closed/shouldsucceed/3054.v b/test-suite/bugs/closed/shouldsucceed/3054.v
new file mode 100644
index 000000000..936e58e19
--- /dev/null
+++ b/test-suite/bugs/closed/shouldsucceed/3054.v
@@ -0,0 +1,10 @@
+Section S.
+
+Let V := Type.
+
+Goal ~ true = false.
+Proof.
+congruence.
+Qed.
+
+End S.