equal
deleted
inserted
replaced
18 typedef ('a, 'b) vec = "UNIV :: ('b::finite \<Rightarrow> 'a) set" |
18 typedef ('a, 'b) vec = "UNIV :: ('b::finite \<Rightarrow> 'a) set" |
19 morphisms vec_nth vec_lambda .. |
19 morphisms vec_nth vec_lambda .. |
20 |
20 |
21 declare vec_lambda_inject [simplified, simp] |
21 declare vec_lambda_inject [simplified, simp] |
22 |
22 |
23 bundle vec_syntax begin |
23 bundle vec_syntax |
24 notation |
24 begin |
25 vec_nth (infixl \<open>$\<close> 90) and |
25 notation vec_nth (infixl \<open>$\<close> 90) and vec_lambda (binder \<open>\<chi>\<close> 10) |
26 vec_lambda (binder \<open>\<chi>\<close> 10) |
26 end |
27 end |
27 |
28 |
28 bundle no_vec_syntax |
29 bundle no_vec_syntax begin |
29 begin |
30 no_notation |
30 no_notation vec_nth (infixl \<open>$\<close> 90) and vec_lambda (binder \<open>\<chi>\<close> 10) |
31 vec_nth (infixl \<open>$\<close> 90) and |
|
32 vec_lambda (binder \<open>\<chi>\<close> 10) |
|
33 end |
31 end |
34 |
32 |
35 unbundle vec_syntax |
33 unbundle vec_syntax |
36 |
34 |
37 text \<open> |
35 text \<open> |