aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/output/SearchPattern.out
diff options
context:
space:
mode:
authorGravatar puech <puech@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-03-11 15:02:49 +0000
committerGravatar puech <puech@85f007b7-540e-0410-9357-904b9bb8a0f7>2010-03-11 15:02:49 +0000
commitb75171fe23f0a0d691961444100710e73e34aa92 (patch)
tree598b58686837767185b5549c91e9afd931d8a1a5 /test-suite/output/SearchPattern.out
parent9da361cdf3e5ee90aa85b0e6432c6cfce5ecb0a5 (diff)
Minimal test suite for search commands
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@12860 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/output/SearchPattern.out')
-rw-r--r--test-suite/output/SearchPattern.out48
1 files changed, 48 insertions, 0 deletions
diff --git a/test-suite/output/SearchPattern.out b/test-suite/output/SearchPattern.out
new file mode 100644
index 000000000..0c32f8d8d
--- /dev/null
+++ b/test-suite/output/SearchPattern.out
@@ -0,0 +1,48 @@
+false: bool
+true: bool
+sumor_beq:
+ forall (A : Type) (B : Prop),
+ (A -> A -> bool) -> (B -> B -> bool) -> A + {B} -> A + {B} -> bool
+sumbool_beq:
+ forall A B : Prop,
+ (A -> A -> bool) -> (B -> B -> bool) -> {A} + {B} -> {A} + {B} -> bool
+xorb: bool -> bool -> bool
+sum_beq:
+ forall A B : Type,
+ (A -> A -> bool) -> (B -> B -> bool) -> A + B -> A + B -> bool
+prod_beq:
+ forall A B : Type,
+ (A -> A -> bool) -> (B -> B -> bool) -> A * B -> A * B -> bool
+orb: bool -> bool -> bool
+option_beq: forall A : Type, (A -> A -> bool) -> option A -> option A -> bool
+negb: bool -> bool
+nat_beq: nat -> nat -> bool
+list_beq: forall A : Type, (A -> A -> bool) -> list A -> list A -> bool
+implb: bool -> bool -> bool
+comparison_beq: comparison -> comparison -> bool
+bool_beq: bool -> bool -> bool
+andb: bool -> bool -> bool
+Empty_set_beq: Empty_set -> Empty_set -> bool
+S: nat -> nat
+O: nat
+pred: nat -> nat
+plus: nat -> nat -> nat
+mult: nat -> nat -> nat
+minus: nat -> nat -> nat
+min: nat -> nat -> nat
+max: nat -> nat -> nat
+length: forall A : Type, list A -> nat
+S: nat -> nat
+pred: nat -> nat
+plus: nat -> nat -> nat
+mult: nat -> nat -> nat
+minus: nat -> nat -> nat
+min: nat -> nat -> nat
+max: nat -> nat -> nat
+mult_n_Sm: forall n m : nat, n * m + n = n * S m
+le_n: forall n : nat, n <= n
+eq_refl: forall (A : Type) (x : A), x = x
+identity_refl: forall (A : Type) (a : A), identity a a
+iff_refl: forall A : Prop, A <-> A
+conj: forall A B : Prop, A -> B -> A /\ B
+pair: forall A B : Type, A -> B -> A * B