aboutsummaryrefslogtreecommitdiffhomepage
path: root/library/library.mllib
diff options
context:
space:
mode:
authorGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-06-29 21:30:19 +0200
committerGravatar Enrico Tassi <Enrico.Tassi@inria.fr>2015-06-29 22:16:07 +0200
commit2defd4c15467736b73f69adb501e3a4fe2111ce5 (patch)
tree6a73e7280956a90e6eb8a588f64a208a3624cd5c /library/library.mllib
parent799f27ae19d6d2d16ade15bbdab83bd9acb0035f (diff)
Assumptions: more informative print for False axiom (Close: #4054)
When an axiom of an empty type is matched in order to inhabit a type, do print that type (as if each use of that axiom was a distinct foo_subproof). E.g. Lemma w : True. Proof. case demon. Qed. Lemma x y : y = 0 /\ True /\ forall w, w = y. Proof. split. case demon. split; [ exact w | case demon ]. Qed. Print Assumptions x. Prints: Axioms: demon : False used in x to prove: forall w : nat, w = y used in w to prove: True used in x to prove: y = 0
Diffstat (limited to 'library/library.mllib')
-rw-r--r--library/library.mllib1
1 files changed, 0 insertions, 1 deletions
diff --git a/library/library.mllib b/library/library.mllib
index eca28c822..920657365 100644
--- a/library/library.mllib
+++ b/library/library.mllib
@@ -16,5 +16,4 @@ Dischargedhypsmap
Goptions
Decls
Heads
-Assumptions
Keys