author | wenzelm |
Wed, 04 Oct 2017 12:00:53 +0200 | |
changeset 66787 | 64b47495676d |
parent 56798 | 939e88e79724 |
child 69605 | a96320074298 |
permissions | -rw-r--r-- |
41561 | 1 |
(* Title: HOL/SPARK/Examples/RIPEMD-160/F.thy |
2 |
Author: Fabian Immler, TU Muenchen |
|
3 |
||
4 |
Verification of the RIPEMD-160 hash function |
|
5 |
*) |
|
6 |
||
7 |
theory F |
|
8 |
imports RMD_Specification |
|
9 |
begin |
|
10 |
||
56798
939e88e79724
Discontinued old spark_open; spark_open_siv is now spark_open
berghofe
parents:
41561
diff
changeset
|
11 |
spark_open "rmd/f" |
41561 | 12 |
|
13 |
spark_vc function_f_2 |
|
14 |
using assms by simp_all |
|
15 |
||
16 |
spark_vc function_f_3 |
|
17 |
using assms by simp_all |
|
18 |
||
19 |
spark_vc function_f_4 |
|
20 |
using assms by simp_all |
|
21 |
||
22 |
spark_vc function_f_5 |
|
23 |
using assms by simp_all |
|
24 |
||
25 |
spark_vc function_f_6 |
|
26 |
proof - |
|
27 |
from H8 have "nat j <= 15" by simp |
|
28 |
with assms show ?thesis |
|
29 |
by (simp add: f_def bwsimps int_word_uint int_mod_eq') |
|
30 |
qed |
|
31 |
||
32 |
spark_vc function_f_7 |
|
33 |
proof - |
|
34 |
from H7 have "16 <= nat j" by simp |
|
35 |
moreover from H8 have "nat j <= 31" by simp |
|
36 |
ultimately show ?thesis using assms |
|
37 |
by (simp add: f_def bwsimps int_word_uint int_mod_eq') |
|
38 |
qed |
|
39 |
||
40 |
spark_vc function_f_8 |
|
41 |
proof - |
|
42 |
from H7 have "32 <= nat j" by simp |
|
43 |
moreover from H8 have "nat j <= 47" by simp |
|
44 |
ultimately show ?thesis using assms |
|
45 |
by (simp add: f_def bwsimps int_word_uint int_mod_eq') |
|
46 |
qed |
|
47 |
||
48 |
spark_vc function_f_9 |
|
49 |
proof - |
|
50 |
from H7 have "48 <= nat j" by simp |
|
51 |
moreover from H8 have "nat j <= 63" by simp |
|
52 |
ultimately show ?thesis using assms |
|
53 |
by (simp add: f_def bwsimps int_word_uint int_mod_eq') |
|
54 |
qed |
|
55 |
||
56 |
spark_vc function_f_10 |
|
57 |
proof - |
|
58 |
from H2 have "nat j <= 79" by simp |
|
59 |
moreover from H12 have "64 <= nat j" by simp |
|
60 |
ultimately show ?thesis using assms |
|
61 |
by (simp add: f_def bwsimps int_word_uint int_mod_eq') |
|
62 |
qed |
|
63 |
||
64 |
spark_end |
|
65 |
||
66 |
end |