src/HOL/SPARK/SPARK.thy
changeset 50788 fec14e8fefb8
parent 47108 2a1953f0d20d
child 54427 783861a66a60
equal deleted inserted replaced
50787:065c684130ad 50788:fec14e8fefb8
   273     with 3 show ?thesis
   273     with 3 show ?thesis
   274       by (simp only: power_BIT mod_BIT int_and_Bits) simp
   274       by (simp only: power_BIT mod_BIT int_and_Bits) simp
   275   qed
   275   qed
   276 qed
   276 qed
   277 
   277 
       
   278 
       
   279 text {* Minimum and maximum *}
       
   280 
       
   281 spark_proof_functions
       
   282   integer__min = "min :: int \<Rightarrow> int \<Rightarrow> int"
       
   283   integer__max = "max :: int \<Rightarrow> int \<Rightarrow> int"
       
   284 
   278 end
   285 end