src/HOL/List.thy
changeset 40077 c8a9eaaa2f59
parent 39963 626b1d360d42
child 40122 1d8ad2ff3e01
equal deleted inserted replaced
40076:6f012a209dac 40077:c8a9eaaa2f59
   260 @{lemma "removeAll 2 [2,0,2,1::nat,2] = [0,1]" by simp}\\
   260 @{lemma "removeAll 2 [2,0,2,1::nat,2] = [0,1]" by simp}\\
   261 @{lemma "nth [a,b,c,d] 2 = c" by simp}\\
   261 @{lemma "nth [a,b,c,d] 2 = c" by simp}\\
   262 @{lemma "[a,b,c,d][2 := x] = [a,b,x,d]" by simp}\\
   262 @{lemma "[a,b,c,d][2 := x] = [a,b,x,d]" by simp}\\
   263 @{lemma "sublist [a,b,c,d,e] {0,2,3} = [a,c,d]" by (simp add:sublist_def)}\\
   263 @{lemma "sublist [a,b,c,d,e] {0,2,3} = [a,c,d]" by (simp add:sublist_def)}\\
   264 @{lemma "rotate1 [a,b,c,d] = [b,c,d,a]" by (simp add:rotate1_def)}\\
   264 @{lemma "rotate1 [a,b,c,d] = [b,c,d,a]" by (simp add:rotate1_def)}\\
   265 @{lemma "rotate 3 [a,b,c,d] = [d,a,b,c]" by (simp add:rotate1_def rotate_def nat_number')}\\
   265 @{lemma "rotate 3 [a,b,c,d] = [d,a,b,c]" by (simp add:rotate1_def rotate_def eval_nat_numeral)}\\
   266 @{lemma "replicate 4 a = [a,a,a,a]" by (simp add:nat_number')}\\
   266 @{lemma "replicate 4 a = [a,a,a,a]" by (simp add:eval_nat_numeral)}\\
   267 @{lemma "[2..<5] = [2,3,4]" by (simp add:nat_number')}\\
   267 @{lemma "[2..<5] = [2,3,4]" by (simp add:eval_nat_numeral)}\\
   268 @{lemma "listsum [1,2,3::nat] = 6" by (simp add: listsum_def)}
   268 @{lemma "listsum [1,2,3::nat] = 6" by (simp add: listsum_def)}
   269 \end{tabular}}
   269 \end{tabular}}
   270 \caption{Characteristic examples}
   270 \caption{Characteristic examples}
   271 \label{fig:Characteristic}
   271 \label{fig:Characteristic}
   272 \end{figure}
   272 \end{figure}