src/HOL/SPARK/Examples/Liseq/Longest_Increasing_Subsequence.thy
changeset 66992 69673025292e
parent 66453 cc19f7ca2ed6
child 69605 a96320074298
equal deleted inserted replaced
66991:fc87d3becd69 66992:69673025292e
     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 Longest_Increasing_Subsequence
     6 theory Longest_Increasing_Subsequence
     7 imports SPARK
     7 imports "HOL-SPARK.SPARK"
     8 begin
     8 begin
     9 
     9 
    10 text \<open>
    10 text \<open>
    11 Set of all increasing subsequences in a prefix of an array
    11 Set of all increasing subsequences in a prefix of an array
    12 \<close>
    12 \<close>