src/HOL/SPARK/Manual/Simple_Greatest_Common_Divisor.thy
changeset 58130 5e9170812356
parent 56798 939e88e79724
child 63167 0909deb8059b
equal deleted inserted replaced
58129:3ec65a7f2b50 58130:5e9170812356
     2     Author:     Stefan Berghofer
     2     Author:     Stefan Berghofer
     3     Copyright:  secunet Security Networks AG
     3     Copyright:  secunet Security Networks AG
     4 *)
     4 *)
     5 
     5 
     6 theory Simple_Greatest_Common_Divisor
     6 theory Simple_Greatest_Common_Divisor
     7 imports SPARK GCD
     7 imports "../SPARK" GCD
     8 begin
     8 begin
     9 
     9 
    10 spark_proof_functions
    10 spark_proof_functions
    11   gcd = "gcd :: int \<Rightarrow> int \<Rightarrow> int"
    11   gcd = "gcd :: int \<Rightarrow> int \<Rightarrow> int"
    12 
    12