aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite
diff options
context:
space:
mode:
authorGravatar vgross <vgross@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-05-31 22:22:10 +0000
committerGravatar vgross <vgross@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-05-31 22:22:10 +0000
commit399777683e67edd649ab26e5b1dde79638f32821 (patch)
tree6120a23faaff1449b38025a468d2141d68535317 /test-suite
parent6b54af467dd9e4e26205e0f16e0c924240fadfe0 (diff)
Introducing strong typing for IDE - toplevel IPC
Obj.magic in toplevel/ide_blob.ml is the only way to simulate GADT. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@13041 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/ide/undo.v1
1 files changed, 1 insertions, 0 deletions
diff --git a/test-suite/ide/undo.v b/test-suite/ide/undo.v
index 84eacc3e3..ea3920551 100644
--- a/test-suite/ide/undo.v
+++ b/test-suite/ide/undo.v
@@ -79,6 +79,7 @@ Definition q := O.
Definition r := O.
(* Bug 2082 : Follow the numbers *)
+(* Broken due to proof engine rewriting *)
Variable A : Prop.
Variable B : Prop.