--- a/src/HOL/Analysis/Finite_Cartesian_Product.thy Tue Feb 20 22:25:23 2018 +0100
+++ b/src/HOL/Analysis/Finite_Cartesian_Product.thy Thu Feb 22 15:17:25 2018 +0100
@@ -20,9 +20,19 @@
declare vec_lambda_inject [simplified, simp]
+bundle vec_syntax begin
notation
vec_nth (infixl "$" 90) and
vec_lambda (binder "\<chi>" 10)
+end
+
+bundle no_vec_syntax begin
+no_notation
+ vec_nth (infixl "$" 90) and
+ vec_lambda (binder "\<chi>" 10)
+end
+
+unbundle vec_syntax
(*
Translate "'b ^ 'n" into "'b ^ ('n :: finite)". When 'n has already more than