src/HOL/SPARK/Manual/Proc2.thy
author wenzelm
Wed, 21 May 2014 22:06:10 +0200
changeset 57051 5e30ffe79980
parent 56798 939e88e79724
child 58130 5e9170812356
permissions -rw-r--r--
spell-checker completion is restricted to explicit mode, to avoid odd effects with immediate edits vs. delayed language context markup, and occasional delays due to dictionary lookup of many variants;

theory Proc2
imports SPARK
begin

spark_open "loop_invariant/proc2"

spark_vc procedure_proc2_7
  by (simp add: ring_distribs pull_mods)

spark_end

end