| author | wenzelm | 
| Tue, 06 Jun 2023 11:07:49 +0200 | |
| changeset 78134 | a11ebc8c751a | 
| parent 69605 | a96320074298 | 
| permissions | -rw-r--r-- | 
| 45044 | 1 | theory Proc2 | 
| 66992 
69673025292e
less global theories -- avoid confusion about special cases;
 wenzelm parents: 
66453diff
changeset | 2 | imports "HOL-SPARK.SPARK" | 
| 45044 | 3 | begin | 
| 4 | ||
| 69605 | 5 | spark_open \<open>loop_invariant/proc2\<close> | 
| 45044 | 6 | |
| 7 | spark_vc procedure_proc2_7 | |
| 64593 
50c715579715
reoriented congruence rules in non-explosive direction
 haftmann parents: 
58130diff
changeset | 8 | by (simp add: ring_distribs mod_simps) | 
| 45044 | 9 | |
| 10 | spark_end | |
| 11 | ||
| 12 | end |