src/HOL/SPARK/Examples/Liseq/Longest_Increasing_Subsequence.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 Longest_Increasing_Subsequence
     6 theory Longest_Increasing_Subsequence
     7 imports SPARK
     7 imports "../../SPARK"
     8 begin
     8 begin
     9 
     9 
    10 text {*
    10 text {*
    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 *}
    12 *}