aboutsummaryrefslogtreecommitdiff
path: root/test-suite
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2020-02-27 15:52:45 -0500
committerEmilio Jesus Gallego Arias2020-02-27 15:52:45 -0500
commitaeca986089d005054496ed4bcf1b920e8fa02173 (patch)
tree074acf720a9969ba3f0d5585edc1351243105fd4 /test-suite
parentc160fc0da9bef60c4ee469cc2c35afd83fc16243 (diff)
parent5ece9623e54ce2a87440c889364c3d1ad5eb52c5 (diff)
Merge PR #11650: Set Printing Parens
Reviewed-by: ejgallego
Diffstat (limited to 'test-suite')
-rw-r--r--test-suite/output/PrintingParentheses.out28
-rw-r--r--test-suite/output/PrintingParentheses.v10
2 files changed, 38 insertions, 0 deletions
diff --git a/test-suite/output/PrintingParentheses.out b/test-suite/output/PrintingParentheses.out
new file mode 100644
index 0000000000..a5874f09a7
--- /dev/null
+++ b/test-suite/output/PrintingParentheses.out
@@ -0,0 +1,28 @@
+((1 + (2 * 3), 4), 5)
+ : (nat * nat) * nat
+mult_n_Sm =
+fun n m : nat =>
+nat_ind (fun n0 : nat => ((n0 * m) + n0) = (n0 * (S m))) eq_refl
+ (fun (p : nat) (H : ((p * m) + p) = (p * (S m))) =>
+ let n0 := p * (S m) in
+ match H in (_ = y) return (((m + (p * m)) + (S p)) = (S (m + y))) with
+ | eq_refl =>
+ eq_ind (S ((m + (p * m)) + p))
+ (fun n1 : nat => n1 = (S (m + ((p * m) + p))))
+ (eq_S ((m + (p * m)) + p) (m + ((p * m) + p))
+ (nat_ind
+ (fun n1 : nat => ((n1 + (p * m)) + p) = (n1 + ((p * m) + p)))
+ eq_refl
+ (fun (n1 : nat)
+ (H0 : ((n1 + (p * m)) + p) = (n1 + ((p * m) + p))) =>
+ f_equal_nat nat S ((n1 + (p * m)) + p)
+ (n1 + ((p * m) + p)) H0) m)) ((m + (p * m)) + (S p))
+ (plus_n_Sm (m + (p * m)) p)
+ end) n
+ : forall n m : nat, ((n * m) + n) = (n * (S m))
+
+Arguments mult_n_Sm (_ _)%nat_scope
+1 :: (2 :: [3; 4])
+ : list nat
+{0 = 1} + {2 <= (4 + 5)}
+ : Set
diff --git a/test-suite/output/PrintingParentheses.v b/test-suite/output/PrintingParentheses.v
new file mode 100644
index 0000000000..190e122e2f
--- /dev/null
+++ b/test-suite/output/PrintingParentheses.v
@@ -0,0 +1,10 @@
+Set Printing Parentheses.
+
+Check (1+2*3,4,5).
+Print mult_n_Sm.
+
+Require Import List.
+Import ListNotations.
+Check [1;2;3;4].
+
+Check {0=1}+{2<=4+5}.